aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* Merge branch 'v8.5' into v8.6Gravatar Pierre-Marie Pédrot2016-07-07
|\
* \ Merge remote-tracking branch 'github/bug4653' into v8.6Gravatar Matthieu Sozeau2016-07-07
|\ \
| | * Prevent "Load" from displaying all the intermediate subgoals.Gravatar Guillaume Melquiond2016-07-07
| | | | | | | | | | | | Note that even "Load Verbose" is not supposed to display them.
| | * Do not display goals in -compile-verbose mode (bug #4841).Gravatar Guillaume Melquiond2016-07-07
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | The -verbose family of options is only meant to echo sentences as they are processed. The patch below broke this, while fixing another issue. That other issue will be fixed in the next commit. Revert "Fixing "Load" without "Verbose" in coqtop, after vernac_com lost its" This reverts commit 2a28c677c3c205ff453b7b5903e4c22f4de2649b.
| * | Do not use implicit type info for (x := t) bindingsGravatar Matthieu Sozeau2016-07-07
| | | | | | | | | | | | | | | | | | This maintains compatibility, it is debatable if we should use implicit type information for lets to allow for coercions to fire. (Problem found in math-comp).
* | | Merge remote-tracking branch 'github/bug4873' into v8.6Gravatar Matthieu Sozeau2016-07-07
|\ \ \
| * | | Program: fix #4873: transparency option not usedGravatar Matthieu Sozeau2016-07-07
|/ / /
| | * Update csdp.cache.Gravatar Maxime Dénès2016-07-06
| | |
| | * Fix typo in configure (noticed by Jason).Gravatar Maxime Dénès2016-07-06
| | |
* | | Merge branch 'primproj' into v8.6Gravatar Matthieu Sozeau2016-07-06
|\ \ \
| * | | Fix reopened bug #3317.Gravatar Matthieu Sozeau2016-07-06
| | | |
| * | | Fixed bug #4622.Gravatar Matthieu Sozeau2016-07-06
| | | |
| * | | Disallow dependent case on prim records w/o etaGravatar Matthieu Sozeau2016-07-06
| | | |
| * | | Renaming to more generic has_dependent_elim testGravatar Matthieu Sozeau2016-07-06
| | | |
| * | | Move is_prim... to Inductiveops and correct SchemeGravatar Matthieu Sozeau2016-07-06
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Now scheme will not try to build ill-typed dependent analyses on recursive records with primitive projections but report a proper error. Minor change of the API (adding one error case to recursion_scheme_error).
| * | | primproj: warning and avoid error.Gravatar Matthieu Sozeau2016-07-06
|/ / / | | | | | | | | | | | | | | | | | | | | | When defining a (co)recursive inductive with primitive projections on, which lacks eta-conversion and hence dependent elimination, build only the associated non-dependent elimination principles, and warn about this. Also make the printing of the status of an inductive w.r.t. projections and eta conversion explicit in Print and About.
| | * Merge remote-tracking branch 'github/pr/199' into v8.5Gravatar Maxime Dénès2016-07-06
| | |\ | | | | | | | | | | | | Was PR#199: Unbreak singleton list-like notation (-compat 8.4)
| | * \ Merge remote-tracking branch 'github/pr/241' into v8.5Gravatar Maxime Dénès2016-07-06
| | |\ \ | | | | | | | | | | | | | | | Was PR#241: Restore option_map in FMapFacts
* | | | | Fix #4793: Coq 8.6 should accept -compat 8.6Gravatar Maxime Dénès2016-07-06
| | | | | | | | | | | | | | | | | | | | We also add a Coq86.v compat file.
| | * | | Bump version number in preparation for 8.5pl2 release.Gravatar Maxime Dénès2016-07-06
| | | | |
| * | | | Fix test-suite file 3690Gravatar Matthieu Sozeau2016-07-06
| | | | |
| | * | | Deduplicate some names in .mailmapGravatar Jason Gross2016-07-06
| | | | |
| * | | | Univs: fix internalization of (x := T) and castsGravatar Matthieu Sozeau2016-07-06
|/ / / / | | | | | | | | | | | | They were allowing algebraic universes to slip in terms.
| * | | Fix indentation of configure printoutGravatar Jason Gross2016-07-06
| | | |
| | * | Move option_map notation upGravatar Jason Gross2016-07-05
| | | | | | | | | | | | This way, it's not eaten by a section
| | * | Restore option_map in FMapFactsGravatar Jason Gross2016-07-05
| |/ / | | | | | | This definition was removed by a4043608f704f026de7eb5167a109ca48e00c221 (This commit adds full universe polymorphism and fast projections to Coq), for reasons I do not know. This means that things like `unfold option_map` work only in 8.5, while `unfold <application of Facts>.option_map` works only in 8.4. This allows `unfold` to work correctly in both 8.4 and 8.5.
| | * Compat84: Don't mess with stdlib modulesGravatar Jason Gross2016-07-05
| | | | | | | | | | | | | | | | | | | | | | | | | | | We don't actually need to, unless we want to support the (presumably uncommon) use-case of someone using [Import VectorNotations] to override their local notation for things in vector_scope. Additionally, we now maintain the behavior that [Import VectorNotations] opens vector_scope.
| * | Prevent unsafe overwriting of Required modules by toplevel library.Gravatar Maxime Dénès2016-07-05
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | In coqtop, one could do for instance: Require Import Top. (* Where Top contains a Definition b := true *) Lemma bE : b = true. Proof. reflexivity. Qed. Definition b := false. Lemma bad : False. Proof. generalize bE; compute; discriminate. Qed. That proof could however not be saved because of the circular dependency check. Safe_typing now checks that we are not requiring (Safe_typing.import) a library with the same logical name as the current one.
| * | congruence fix: test-suite code and update CHANGESGravatar Matthieu Sozeau2016-07-05
| | | | | | | | | | | | This fixes bugs #4069 (not 4609 as mentionned in the git log) and #4718.
* | | Revert "Merge remote-tracking branch 'github/pr/229' into trunk"Gravatar Maxime Dénès2016-07-05
| | | | | | | | | | | | | | | | | | | | | | | | | | | This reverts commit b2f8f9edd5c1bb0a9c8c4f4b049381b979d3e385, reversing changes made to da99355b4d6de31aec5a660f7afe100190a8e683. Hugo asked for more discussion on this topic, and it was not in the roadmap. I merged it prematurely because I thought there was a consensus. Also, I missed that it was changing coq_makefile. Sorry about that.
| * | Pass .v files to coqc in Makefile produced by coq_makefile (bug #4896).Gravatar Guillaume Melquiond2016-07-05
| | | | | | | | | | | | | | | Coqc now expects physical names for input files, so fix coq_makefile accordingly.
| * | Add mailmap entry.Gravatar Guillaume Melquiond2016-07-05
| | |
| * | Bug fix : variable capture in ltac code of NsatzGravatar thery2016-07-05
| | | | | | | | | | | | | | | | | | | | | | | | changing set (x := val) into let x := fresh "x" in set (x := val)
* | | FIX: "dev/doc/changes.txt"Gravatar Matej Kosik2016-07-05
| | |
* | | Merge remote-tracking branch 'github/pr/229' into trunkGravatar Maxime Dénès2016-07-04
|\ \ \ | | | | | | | | | | | | Was PR#229: Bytecode compilation in a new 'make byte' rule apart from 'make world'
| | * \ Merge branch 'congruencefix' into v8.5Gravatar Matthieu Sozeau2016-07-04
| | |\ \
* | | | | Revert "Revert "Improve the interpretation scope of arguments of an ltac ↵Gravatar Maxime Dénès2016-07-04
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | match."" We apply this patch to trunk so that it is integrated in 8.6. This reverts commit 0eb08b70f0c576e58912c1fc3ef74f387ad465be.
* | | | | Merge branch 'v8.5' into trunkGravatar Maxime Dénès2016-07-04
|\ \ \ \ \ | | |/ / / | |/| | |
| | | * | congruence: Restrict refreshing to SetGravatar Matthieu Sozeau2016-07-04
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | Because refreshing Prop is not semantics-preserving, the new universe is >= Set, so cannot be minimized to Prop afterwards.
| | | * | congruence: remove casts of indexed termsGravatar Matthieu Sozeau2016-07-04
| | | | | | | | | | | | | | | | | | | | | | | | | This fixes the end of bug #4069, provoked by a use of unshelve refine which introduces a cast.
| | | * | congruence/univs: properly refresh (fix #4609)Gravatar Matthieu Sozeau2016-07-04
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | In congruence, refresh universes including the Set/Prop ones so that congruence works with cumulativity, not restricting itself to the inferred types of terms that are manipulated but allowing them to be used at more general types. This fixes bug #4609.
* | | | | Update CHANGES, the bugfixes for 4527 and 4726 areGravatar Matthieu Sozeau2016-07-04
| | | | | | | | | | | | | | | | | | | | not in pl2.
| * | | | Mention more fixes in CHANGES before we release pl2.Gravatar Maxime Dénès2016-07-04
| | | | |
| * | | | Revert "Improve the interpretation scope of arguments of an ltac match."Gravatar Maxime Dénès2016-07-04
| | |/ / | |/| | | | | | | | | | | | | | | | | | We apply this patch to trunk for integration in 8.6 instead. This reverts commit 715f547816addf3e2e9dc288327fcbcee8c6d47f.
| * | | test-suite: test checking of libraries checksum.Gravatar Maxime Dénès2016-07-04
| | | |
| * | | Merge remote-tracking branch 'github/pr/228' into v8.5Gravatar Maxime Dénès2016-07-04
| |\ \ \ | | | | | | | | | | | | | | | | | | | | | | | | | Was PR#228: fix coqide double module linking (error on OCaml 4.03) Fixes #4747: Problem building Coq 8.5pl1 with OCaml 4.03.0: Fatal warnings triggered by CoqIDE
* | | | | Remove lexing of ordinal notations.Gravatar Maxime Dénès2016-07-03
| | | | | | | | | | | | | | | | | | | | | | | | | This was implemented in anticipation of a part of PR#164 that we decided not to merge.
* | | | | Mention recent renaming of files in dev/doc/changes.txt.Gravatar Maxime Dénès2016-07-03
| | | | |
* | | | | Merge branch 'cerrors-cclosure' into trunkGravatar Maxime Dénès2016-07-03
|\ \ \ \ \ | | | | | | | | | | | | | | | | | | Was PR#226: CErrors & CClosure
| * | | | | rename toplevel/cerror.ml into explainErr.ml (too close to the new ↵Gravatar Pierre Letouzey2016-07-03
| | | | | | | | | | | | | | | | | | | | | | | | lib/cErrors.ml)