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

Fix #18351

needs: fixing
kind: enhancement
part: ltac2
needs: full CI

cf #10556 The previous behaviour can be gotten by doing eg ~~~coq (* auxiliary definition to avoid repeating it, if it's a simple expression it can also be inlined *)...

part: ltac2

We move the code responsible from the generation of the forcing of lazy constants in the native compiler to the second compilation phase. This also has the nice side-effect of...

kind: cleanup

This is an experimental PR propagating the unfolded status of primitive projections to parsing and printing so that special parsing/printing notations can be used to refer to them. In the...

needs: rebase
part: primitive records
part: parser
part: printer
stale
needs: full CI

See discussion at coq/ceps#42. We introduce `Body` as a synonymous of `Proof` to delimit the beginning of a definition by tactics. When used in the form `Body c`, it indicates...

needs: discussion
kind: enhancement
kind: usability
needs: full CI

Quick and dirty experiment following the Coq call. Rather than implementing a full-blown refolding of fixpoint everywhere, we experiment with refolding when converting only.

needs: rebase

```coq (* coqc -native-compiler yes bar.v *) Fixpoint fact n := match n with S n' => n * fact n' | O => 1 end. Definition large : nat...

part: native compiler
kind: bug

This pull request implements the proposal in issue #18212 . The documentation markup files are already updated accordingly. I am very open for remarks and critics and I hope that...

kind: feature
part: extraction
needs: full CI

Hello. Thank you for providing such good libre software. This week, I’ve worked on improving the UI of CoqIDE, especially the Preferences dialog. Indeed, I’ve started to use CoqIDE at...

needs: rebase
needs: full CI