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

### Is your feature request related to a problem? In classes, it is often the case that we want to show multiple proofs of the same lemma. At this point,...

kind: feature
needs: triage
kind: wish
kind: design discussion

The goal is to be able to detect bugs like https://github.com/coq/coq/issues/20224 so we don't want to just check that all templates are fully applied. Instead we keep around a set...

kind: user messages

VERNAC EXTEND doc should be reasonably complete with this. We could also consider promoting parsing.md to a refman page.

kind: documentation

### Description of the problem I think there is an issue with the reverse coercion mechanism. Take: - `A1` (reverse) coercible to class `C` through class `B`, with the coercion...

needs: progress
kind: bug

Depends: - https://github.com/rocq-prover/rocq/pull/20542

needs: progress
kind: feature
needs: rebase
part: ltac2
needs: full CI

Errors: ``` logs/primitive/arrays/get.v.log ==========> TESTING primitive/arrays/get.v t.[0] : forall A : Type, array A -> A fun (A : Type) (t : array A) => t.[0] : forall A :...

part: VM

If: - coercion class `A1` is (reverse) coercible to class `C` through class `B`, with the coercion between `A1` and `B` an identity coercion `id_A1`; - coercion class `A2` is...

needs: discussion

### Description of the problem ``` COQPATH=$PWD rocq repl -w -deprecated-coq-env-var Warning, feedback message received but no listener to handle it! Warning, feedback message received but no listener to handle...

kind: user messages
kind: bug

The PR makes a minimal modification to the proof-search of `tauto` so that `axioms` are checked for each time a new formula is generated. + This may avoid performing a...

needs: fixing
kind: performance
kind: enhancement
needs: benchmarking

### Description of the problem The `Combined Scheme` is very inconsistent and sometimes crashes. Several examples: ```coq Inductive A := a : A with B := b : B. Scheme...

kind: bug
needs: triage