coq
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...
Fix #18351
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 *)...
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...
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...
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...
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.
```coq (* coqc -native-compiler yes bar.v *) Fixpoint fact n := match n with S n' => n * fact n' | O => 1 end. Definition large : nat...
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...
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...