aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* [configure] 'ocaml' is more precise than OCaml as we mean the binary.Gravatar Maxime Dénès2017-06-23
| | | | Fix suggested by Hugo.
* ocaml -> OCaml in configure.ml.Gravatar Maxime Dénès2017-06-23
|
* Merge PR#729: Fixing an inconsistency between configure and configure.mlGravatar Maxime Dénès2017-06-23
|\
* \ Merge PR#740: Refactor documentation of records.Gravatar Maxime Dénès2017-06-23
|\ \
* \ \ Merge PR#812: Use more neutral wording instead of mentioning CoqIDEGravatar Maxime Dénès2017-06-20
|\ \ \
* \ \ \ Merge PR#792: Fix ci-fiat-crypto to have a proper lite targetGravatar Maxime Dénès2017-06-19
|\ \ \ \
| | * | | Change CoqIDE-specific to neutral wordingGravatar Paul Steckler2017-06-19
| |/ / / |/| | |
| * | | Remove -j ${NJOBS} from make invocations in the ciGravatar Jason Gross2017-06-16
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | According to https://www.gnu.org/software/make/manual/html_node/Options_002fRecursion.html#Options_002fRecursion it's not necessary, because we pass `-j ${NJOBS}` to the top-level `make` invocation in `.travis.yml`. Additionally, explicitly passing `-j` in, e.g., fiat-crypto, results in error messages such as ``` make[2]: *** write jobserver: Bad file descriptor. Stop. make[2]: *** Waiting for unfinished jobs.... make[2]: *** write jobserver: Bad file descriptor. Stop. make[1]: *** [coqprime] Error 2 make[1]: INTERNAL: Exiting with 1 jobserver tokens available; should be 2! make[1]: Leaving directory `/home/travis/build/JasonGross/coq/_build_ci/fiat-c ``` because the `-j` on the `make` in the `ci-fiat-crypto.sh` script disables jobserver mode, and the submake in fiat-crypto to make coqprime does not explicitly pass `-j`, and so reenables jobserver mode, and then `make` gets very confused. Commit made with ```bash cd dev/ci git grep --name-only -- 'make -j ${NJOBS}' | xargs sed s'/make -j \${NJOBS}/make/g' -i git grep --name-only -- 'make -f Makefile.coq -j ${NJOBS}' | xargs sed s'/make -f Makefile.coq -j \${NJOBS}/make -f Makefile.coq/g' -i ```
| * | | Pass GNU Make jobserver on to the ci jobsGravatar Jason Gross2017-06-16
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Solution found by reading the question [Is it possible to “pass-through” GNU make jobserver environment to a submake served via a 3rd-party (non-make)](https://stackoverflow.com/q/29910944/377022). This, I hope, will fix errors such as ``` make[2]: *** write jobserver: Bad file descriptor. Stop. make[2]: *** Waiting for unfinished jobs.... make[2]: *** write jobserver: Bad file descriptor. Stop. make[1]: *** [coqprime] Error 2 make[1]: INTERNAL: Exiting with 1 jobserver tokens available; should be 2! make[1]: Leaving directory `/home/travis/build/JasonGross/coq/_build_ci/fiat-c ``` which result from having a top-level `make` which sets up the jobserver (via `-jN`), which invokes a non-makefile script *without passing on the file descriptors for the jobserver*, which either invokes a makefile script without `-jN` or invokes a makefile script with `-jN` which itself invokes a submake without `-jN`. This was the case, for example, in fiat-crypto.
| * | | Fix ci-fiat-crypto to have a proper lite targetGravatar Jason Gross2017-06-16
|/ / / | | | | | | | | | | | | The lite target depends on having the submodule cloned to generate the list of files to not build.
* | | Merge PR#730: Protecting from warnings while compiling 8.6Gravatar Maxime Dénès2017-06-16
|\ \ \
| | * | Refactor documentation of records.Gravatar Théo Zimmermann2017-06-16
| | | | | | | | | | | | | | | | This fixes bug https://coq.inria.fr/bugs/show_bug.cgi?id=4971
* | | | Merge PR#767: Document named evars (including Show ident)Gravatar Maxime Dénès2017-06-16
|\ \ \ \
* \ \ \ \ Merge PR#741: Fix documentation of Typeclasses eauto :=Gravatar Maxime Dénès2017-06-15
|\ \ \ \ \
* \ \ \ \ \ Merge PR#713: Bump year in headers.Gravatar Maxime Dénès2017-06-15
|\ \ \ \ \ \
* \ \ \ \ \ \ Merge PR#440: Univs: fix bug #5365, generation of u+k <= v constraintsGravatar Maxime Dénès2017-06-15
|\ \ \ \ \ \ \
* \ \ \ \ \ \ \ Merge PR#752: Adding a test case as requested in bug 5205.Gravatar Maxime Dénès2017-06-15
|\ \ \ \ \ \ \ \
* \ \ \ \ \ \ \ \ Merge PR#747: Fix Bug #5568, no dup notation warnings on repeated module importsGravatar Maxime Dénès2017-06-15
|\ \ \ \ \ \ \ \ \ | |_|_|_|_|_|_|/ / |/| | | | | | | |
| | | | | | * | | Document instantiate (ident := term) and make it the preferred variant.Gravatar Théo Zimmermann2017-06-13
| | | | | | | | |
| | | | | | * | | Document Show ident.Gravatar Théo Zimmermann2017-06-13
| | | | | | | | |
| | | | | | * | | Document evar naming syntax.Gravatar Théo Zimmermann2017-06-13
| |_|_|_|_|/ / / |/| | | | | | |
| * | | | | | | Fix Bug #5568, no dup notation warnings on repeated module importsGravatar Paul Steckler2017-06-09
| | | | | | | |
| | * | | | | | Adding a test case as requested in bug 5205.Gravatar Théo Zimmermann2017-06-08
| |/ / / / / / |/| | | | | |
| | | | * | | Fix documentation of Typeclasses eauto :=Gravatar Théo Zimmermann2017-06-07
| |_|_|/ / / |/| | | | |
| | * | | | Univs: fix bug #5365, generation of u+k <= v constraintsGravatar Matthieu Sozeau2017-06-05
| | | | | | | | | | | | | | | | | | | | | | | | Use an explicit label ~algebraic for make_flexible_variable as well.
| | | | * | Ensure that warnings new from ocaml > 4.01 remains silent.Gravatar Hugo Herbelin2017-06-04
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Indeed, 8.6 is announced to be compilable with 4.01.0 and it is convenient not seeing warnings about which nothing can be done. Remove deprecation warnings new from ocaml 4.03, as well as warning 52. This is a partial cherry-pick of a77734ad6.
| | | | * | configure: avoid deprecated warningsGravatar Pierre Letouzey2017-06-04
| |_|_|/ / |/| | | |
| | | | * Fixing an inconsistency between configure and configure.ml.Gravatar Hugo Herbelin2017-06-04
| |_|_|/ |/| | | | | | | | | | | | | | | The shell script configure was assuming the existence of option -camldir which was removed in 333d41a9.
* | | | Merge PR#705: Fix bug #5019 (looping zify on dependent types)Gravatar Maxime Dénès2017-06-02
|\ \ \ \ | |/ / / |/| | |
* | | | Merge PR#631: Fix bug #5255Gravatar Maxime Dénès2017-06-01
|\ \ \ \
| | | | * Bump year in headers.Gravatar Maxime Dénès2017-06-01
| | | | |
| | * | | Fix bug #5019 (looping zify on dependent types)Gravatar Jason Gross2017-06-01
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | This fixes [bug #5019](https://coq.inria.fr/bugs/show_bug.cgi?id=5019), "[zify] loops on dependent types"; before, we would see a `Z.of_nat (S ?k)` which could not be turned into `Z.succ (Z.of_nat k)`, add a hypothesis of the shape `0 <= Z.of_nat (S k)`, turn that into a hypothesis of the shape `0 <= Z.succ (Z.of_nat k)`, and loop forever on this. This may not be the "right" fix (there may be cases where `zify` should succeed where it still fails with this change), but this is a pure bugfix in the sense that the only places where it changes the behavior of `zify` are the places where, previously, `zify` looped forever.
| | * | | Add opened bug 5019Gravatar Jason Gross2017-06-01
| | | | |
* | | | | Merge PR#710: Add test-suite checks for coqchk with constraintsGravatar Maxime Dénès2017-06-01
|\ \ \ \ \ | |_|/ / / |/| | | |
* | | | | Merge PR#560: Reinstate fixpoint refolding in [cbn], deactivated by mistake ↵Gravatar Maxime Dénès2017-05-31
|\ \ \ \ \ | | | | | | | | | | | | | | | | | | (EDIT: for mutual fixpoints)
* \ \ \ \ \ Merge PR#699: Fix bug 5550: "typeclasses eauto with" does not work with ↵Gravatar Maxime Dénès2017-05-31
|\ \ \ \ \ \ | |_|_|_|_|/ |/| | | | | | | | | | | section variables.
| | | * | | Add test-suite checks for coqchk with constraintsGravatar Jason Gross2017-05-30
| |_|/ / / |/| | | |
* | | | | Merge PR#693: A subtle bug in tclWITHHOLES.Gravatar Maxime Dénès2017-05-30
|\ \ \ \ \
* \ \ \ \ \ Merge PR#695: Omega: fix bug #4132Gravatar Maxime Dénès2017-05-30
|\ \ \ \ \ \
| | | * | | | Fix bug 5550: "typeclasses eauto with" does not work with section variables.Gravatar Théo Zimmermann2017-05-30
| |_|/ / / / |/| | | | |
| * | | | | Omega: use "simpl" only on coefficents, not on atoms (fix #4132)Gravatar Pierre Letouzey2017-05-29
|/ / / / / | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Two issues in one: - some focused_simpl were called on the wrong locations - some focused_simpl were done on whole equations In the two cases, this could be bad if "simpl" goes too far with respect to what omega expects: later calls to "occurrence" might fail. This may happen for instance if an atom isn't a variable, but a let-in (b:=5:Z in the example).
* | | | | Merge PR#685: Fix a bug in checkerGravatar Maxime Dénès2017-05-29
|\ \ \ \ \
* \ \ \ \ \ Merge PR#546: Fix for bug #4499 and other minor related bugsGravatar Maxime Dénès2017-05-29
|\ \ \ \ \ \
| | * | | | | Fix a bug in checkerGravatar Amin Timany2017-05-28
| |/ / / / / |/| | | | | | | | | | | | | | | | | Universe constraints of the inductive types were not instantiated before being pushed on the environment. This commit fixes this bug.
| | * | | | Fixing a subtle bug in tclWITHHOLES.Gravatar Hugo Herbelin2017-05-28
| |/ / / / |/| | | | | | | | | | | | | | This fixes Théo's bug on eset.
* | | | | Merge PR#679: Bug 5546, qualify datatype constructors when needed in Show MatchGravatar Maxime Dénès2017-05-28
|\ \ \ \ \
* \ \ \ \ \ Merge PR#634: Fix bug #5526, don't check for nonlinearity in notation if ↵Gravatar Maxime Dénès2017-05-26
|\ \ \ \ \ \ | | | | | | | | | | | | | | | | | | | | | printing only
* \ \ \ \ \ \ Merge PR#672: Add parsers-examples target to fiat-parsers ciGravatar Maxime Dénès2017-05-26
|\ \ \ \ \ \ \
| | | * | | | | Bug 5546, qualify datatype constructors when neededGravatar Paul Steckler2017-05-25
| | | | | | | |
* | | | | | | | Merge PR#416: Fix the way setoid_rewrite handles bindings.Gravatar Maxime Dénès2017-05-25
|\ \ \ \ \ \ \ \ | |_|_|/ / / / / |/| | | | | | |