-
```
Section A.
Variable NOTUSED: nat.
Theorem trivial_lemma: 0 = 0.
Proof.
auto.
Qed.
End A.
```
In this code, the type of `trivial_lemma` outside the section `A` is `tr…
-
The “rewrite” tactic from SSReflect (and probably other tactics that perform some matching) fails at inferring a canonical instance when the symbol that triggers the resolution is a primitive projecti…
-
Does it make sense to move [`unit_irrelevance`](https://github.com/math-comp/finmap/blob/92a959e9e91ca356b937923bc823c7f7bb9029b5/order.v#L290) elsewhere in Coq's part of ssreflect or mathcomp?
E.g…
-
### Description of the problem
Assumption interpretation (i.e., `move => /foo`) fails on trivial examples. The equivalent construction in vanilla Ltac (i.e., `intros H%foo`) works fine, as does the f…
-
In the current version of the library, inversion on formulas is not working as expected. In some cases, for instance, `congruence` falls short of closing a goal `s = t` given the assumption `q → s = q…
-
When running a Coq file produces warnings, PG will show these warnings in the bottom-right window, but there is no way (that I could find) to figure out which lines the warning are talking about. To r…
-
Hello,
I am using the electric terminator mode and I have "Proof Next Command Insert Space" enabled but when I enter a terminator ('.' in coq) PG moves the cursor ('|' in the example below) to the b…
-
#### Version
8.8
#### Operating system
Linux
#### Description of the problem
The following produces a term that fails to typecheck at Qed:
```coq
Variable F : Prop -> Prop.
Variabl…
-
in 8.13.2:
```Coq
From Coq Require Import Logic.StrictProp.
Parameter foo: sEmpty -> nat.
Goal forall (a b:sEmpty), foo a = foo b.
intros a b. Fail congruence. reflexivity.
Qed.
```
-
```
Windows STD_INT > vc 6
http://www.azillionmonkeys.com/qed/pstdint.h
```
Original issue reported on code.google.com by `0xcafef...@gmail.com` on 1 Jun 2011 at 12:24