coq icon indicating copy to clipboard operation
coq copied to clipboard

Coq is a formal proof management system. It provides a formal language to write mathematical definitions, executable algorithms and theorems together with an environment for semi-interactive developme...

Results 720 coq issues
Sort by recently updated
recently updated
newest added

As @herbelin said [here](https://github.com/coq/coq/pull/19475#pullrequestreview-2278374479): > On the other side, I'm unsure we have to be proud that cyclic equalities are not automatically found contradictory. If not by `discriminate`, there should...

part: tactics
good first issue
kind: enhancement
kind: wish

### Description of the problem I write a Coq project managing a lot of list equalities containing `++`. To simplify rewriting hypothesis into such list equalities, I use a package...

kind: bug
needs: triage

### Is your feature request related to a problem? Tactic `discriminate` is able to refutes `S n = 0` and it does it by mapping `S n` to `True` and...

kind: wish
part: inversion tactics

### Description of the problem the `discriminate` and `injection` tactics are not compatible with sort polymorphic inductive types instantiated at `Type` ### Small Coq file to reproduce the bug ```coq...

kind: bug
needs: triage

Since #16931 , `./configure -bytecode-compiler no` had no effect, as we stopped checking the flag. We do instead like native and set default options flag. I wonder if these options...

kind: bug
needs: full CI

### Description of the problem Consider this little example: ~~~coq From Coq Require Import FinFun. From Coq Require Import Classes.Equivalence. Definition f_id {X: Type} (x0: X) := x0. Lemma simpl_prop:...

kind: bug

~~~coq (* -*- coq-prog-args: ("-impredicative-set"); -*- *) Inductive X : Set := x : Type -> bool -> X. Goal x bool true x bool false. red. Fail discriminate. injection....

kind: bug
part: inversion tactics

### Description of the problem `induction IHm` drops `IHm` from the context. It should give a error and make no change if that's not too hard. ![image](https://github.com/user-attachments/assets/3ac81937-6f97-4ade-8194-4114ef720395) ### Small Coq...

part: tactics
kind: bug
needs: triage

### Description of the problem Between `8.20.0` and current `8.21+alpha` for (to me) unclear reasons there are universe inconsistencies in [coq-library-undecidability](https://github.com/uds-psl/coq-library-undecidability/tree/master). ### Small Coq file to reproduce the bug ```coq...

kind: regression
part: universes
kind: bug

So the URL is https://coq.inria.fr/doc/v8.19/refman/ instead of https://coq.inria.fr/doc/V8.19.2/refman/ also https://coq.inria.fr/doc/v8.19/refman/changes.html has an "unreleased changes" section at the beginning Is using the branch deliberate?