-
When using macros in action facts in lemmas like in the following theory
```
theory MacrosInActions
begin
macros:
m(x) = x
rule A:
[ In(x) ] --[ A(m(x)) ]-> [ ]
lemma M:
exist…
-
When rewriting a lemma with exponents it takes a long time to finish. The problem occurs both in `rewrite bound` and `rewrite (ltz_trans ....)`.
```ocaml
require import AllCore IntDiv.
op p1:in…
-
We should standardize these and enforce in the validator. As is, e.g. "its" is sometimes lemmatized as "it".
The UD lemmatization policies have evolved and are summarized [here for pronouns](https:…
-
In this module, we have a lemma `hardpost` whose spec is "hard" to verify (in this case, it's actually incorrect, so this example is not brittle). After verifying it, in this case just admitting it, w…
-
Came across a few words where the lemmas are apparently one of two options. This is a little inconvenient in terms of learning how to lemmatize German. Is there a way to unify these? For example, t…
-
There is a second identity in this space; we currently only have proven one:
```lean4
x >>> n n := by
```
Also, what about sshiftRight?
-
Hi,
thank you all for agda-categories :-) I spent almost entire last year on an initial F-algebra construction, which builds the initial algebra from finite, recursive F-coalgebras ("Initial Algebr…
-
[Wiktionary - Category:Coptic lemmas](https://en.wiktionary.org/wiki/Category:Coptic_lemmas)
-
These involve counting the number of equations up to relabeling and relabeling + symmetry, they involve the Catalan numbers and the [Bell numbers](https://en.wikipedia.org/wiki/Bell_number) which AFAI…
-
Now that we have abelian categories in #1929, its time to think about how we can go proving various items in the toolbox of homological algebra.
We can prove the short 5-lemma and then the rest, bu…