-
#### Description of the problem
In the following code:
```coq
Ltac introsuntil h := intros until h.
Goal forall t : nat, t = t.
Proof.
introsuntil t.
reflexivity.
Qed.
Require Imp…
-
```
$ cat toBeautify.v
```
```
Inductive Foo := Foo1 | Foo2 | Foo3.
Definition isFoo12(f: Foo): bool :=
match f with
| Foo1 => true
| Foo2 => true
| _ => false
end.
```
```…
-
#### Description of the problem
`typeclasses eauto` may fail on a trivial goal, whereas `typeclasses eauto with nocore` succeeds (using stronger unification).
```coq
Create HintDb empty.
Goa…
-
#### Description of the problem
The `rewrite` in the following example fails:
```coq
Set Primitive Projections.
Record R := { n : nat; }.
Lemma uhh (r : R) (H : n r = 0) :
n r = 0.
Proo…
-
Hello, I just learned about this project and Globular. It's really exciting to see a proof assistant for HoTT!
It would be valuable to see some example proofs for those of us who are coming from a …
-
#### Description of the problem
Require Import Recdef.
Class C := { }.
Function f `{C} (l : list nat) {measure length l} := l.
Error:
Anomaly "File "plugins/funind/gen_principle.ml", line 166…
-
#### Description of the problem
```coq
Require Import Coq.Program.Tactics.
Record Progression : Type := {
next: Set;
}.
Existing Class Progression.
#[export, program]
Instance item_l…
-
Coq is a proof assistant that allows users to write and verify mathematical proofs using a formal language called Gallina. Ltac is a tactic language for Coq, which enables users to automate parts of t…
-
#### Description of the problem
The first `nia` below fails on Coq 8.11.0 but works on Coq 8.10.2.
```
Require Import Lia.
Goal forall k1 k2 R1 R2,
k1 < 1 -> k2 < R1 + R2 ->
k1 * (R1…
-
Will it be possible to support logos of https://coq.inria.fr/ and https://agda.readthedocs.io/en/v2.6.1.3/ ?
They are both quite famous proof assistants, so it will be great if the support is possibl…