aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* Native compiler: refactor code handling pre-computed values.Gravatar Maxime Dénès2015-07-10
| | | | Fixes #4139 (Not_found exception with Require in modules).
* Kernel/Checker: Cleanup fixes of substitutions due to let-ins.Gravatar Matthieu Sozeau2015-07-09
| | | | | Avoid undeeded large substitutions, and add test-suite file for fixed bug 4283 in closed/
* Kernel: primitive projections handling of let-insGravatar Matthieu Sozeau2015-07-09
| | | | | | | Fixes bug #4176 (actually two bugs in one) Correct computation of the type of primitive projections in presence of let-ins.
* Improve semantics of -native-compiler flag.Gravatar Maxime Dénès2015-07-09
| | | | | | | | | | Since Guillaume's, launching coqtop without -native-compiler and call native_compute would mean recompiling silently all dependencies, even if they had been precompiled (e.g. the stdlib). The new semantics is that -native-compiler disables separate compilation of the current library, but still tries to load precompiled dependencies. If loading fails when the flag is on, coqtop stays silent.
* Template polymorphism: A bug-fix for Bug #4258Gravatar mlasson2015-07-09
| | | | | | | | | | | Reviewed by M. Sozeau This commit fixes template polymorphism and makes it more precise, applying to non-linear uses of the same universe in parameters of template-polymorphic inductives. See bug report and https://github.com/coq/coq/pull/69 for full details. I also removed some deadcode in checker/inductive.ml. I do not know if it is also necessary to fix checker/indtypes.ml.
* Make retyping of projections more resilient to wrong environment.Gravatar Maxime Dénès2015-07-09
| | | | | | Unfortunately, it seems that retyping can be called in ill-typed terms and/or in the wrong environment. This was broken for projections by my commit a51cce369b9c634a93120092d4c7685a242d55b1
* Fixing printing of primitive coinductive record status.Gravatar Pierre-Marie Pédrot2015-07-09
| | | | They do not have eta-rule indeed, even though it was displayed as such.
* Ide: fix bug #4284 for goodGravatar Matthieu Sozeau2015-07-08
| | | | Correct folding order over the named_list_context.
* Bug 4284: Tentative bugfix for detyping exception.Gravatar Matthieu Sozeau2015-07-08
|
* Checker: Report bugfixes from kernel/inductive.mlGravatar Matthieu Sozeau2015-07-08
| | | | Wrong handling of mind_params_ctxt...
* Fix documentation of universes.Gravatar Matthieu Sozeau2015-07-08
|
* Make sure that scope classes are displayed by Print Scopes. (Fix bug #4262)Gravatar Guillaume Melquiond2015-07-08
|
* Fix command-line documentation of coq-tex.Gravatar Guillaume Melquiond2015-07-08
|
* Fix documentation.Gravatar Guillaume Melquiond2015-07-08
|
* Use the same optimization level for the VM, whatever the debug level.Gravatar Guillaume Melquiond2015-07-08
|
* Document Set/Print Firstorder Solver option.Gravatar Matthieu Sozeau2015-07-07
|
* Checker: Fix bug #4282Gravatar Matthieu Sozeau2015-07-07
| | | | | Adapt to new [projection] abstract type comprising a constant and a boolean.
* Univs: bug fix.Gravatar Matthieu Sozeau2015-07-07
| | | | | Missing universe substitutions of mind_params_ctxt when typechecking cases, which appeared only when let-ins were used.
* test-suite: Fix test-suite MakefileGravatar Matthieu Sozeau2015-07-07
| | | | | Using relative path for coqlib, for some reason this fails on Mac OS X. Took the easiest way to fix it.
* Univs/minimization: Fix unused variable bug.Gravatar Matthieu Sozeau2015-07-07
|
* Fixing "Load" without "Verbose" in coqtop, after vernac_com lost itsGravatar Hugo Herbelin2015-07-07
| | | | verbose flag.
* Test case for #4203, fixed by commit a51cce36.Gravatar Maxime Dénès2015-07-06
|
* Fixing documentation (see Maxime's mail on coqdev, July 3).Gravatar Hugo Herbelin2015-07-05
|
* More precise rewording about asymmetric patterns.Gravatar Hugo Herbelin2015-07-05
|
* Fix handling of primitive projections in VM.Gravatar Maxime Dénès2015-07-05
| | | | | I'm pushing this patch now because the previous treatment of such projections in the VM was already unsound. It should however be carefully reviewed.
* Fixing bug #4265: coqdep does not handle From ... Require.Gravatar Pierre-Marie Pédrot2015-07-03
| | | | | | The search algorithm is not satisfactory though, as it crawls through all known files to find the proper one. We should rather use some trie-based data structure, but I'll leave this for a future commit.
* Fix convertibility of primitive projections for native_compute.Gravatar Maxime Dénès2015-07-03
| | | | Stuck primitive projections were never convertible.
* More robust pattern matching on structured constants in VM.Gravatar Maxime Dénès2015-07-02
|
* Revert "Add target to install dev files."Gravatar Maxime Dénès2015-07-02
| | | | | | Broke the build. This reverts commit ef6459b00999a29183edc09de9035795ff7912e9.
* Fix loop in assumptions (Close: #4275)Gravatar Enrico Tassi2015-07-02
|
* Display functions for primitive projections.Gravatar Maxime Dénès2015-07-02
|
* Further simplification of the graph traversal in Univ.Gravatar Pierre-Marie Pédrot2015-07-01
| | | | | | | | We passed the arc to be marked as visited to the functions pushing the neighbours on the remaining stack, but this can be actually done before pushing them, as the [process_le] and [process_lt] functions do not rely on the visited flag. This exposes more clearly the invariants of the algorithm.
* Notation: use same level for "@" in constr: and pattern: (Close: #4272)Gravatar Enrico Tassi2015-07-01
| | | | | | | A possible script breakage can occur if one has a notation at level 11 that is also right associative (now 11 is left associative). Thanks Georges for debugging that.
* Removing dead code in coqdep.Gravatar Pierre-Marie Pédrot2015-06-30
| | | | | | Since commit 2f521670fbd, the Require "file" syntax was not used anymore by coqtop but the code handling it was still there in coqdep. We finish the work by erasing the remnant code.
* Assumptions: more informative print for False axiom (Close: #4054)Gravatar Enrico Tassi2015-06-29
| | | | | | | | | | | | | | | | | | | | | | | | When an axiom of an empty type is matched in order to inhabit a type, do print that type (as if each use of that axiom was a distinct foo_subproof). E.g. Lemma w : True. Proof. case demon. Qed. Lemma x y : y = 0 /\ True /\ forall w, w = y. Proof. split. case demon. split; [ exact w | case demon ]. Qed. Print Assumptions x. Prints: Axioms: demon : False used in x to prove: forall w : nat, w = y used in w to prove: True used in x to prove: y = 0
* class_tactics: make interruptibleGravatar Enrico Tassi2015-06-29
| | | | Tracing with gdb by Alec Faithfull
* class_tactics: remove catch-all, use Errors.noncriticalGravatar Enrico Tassi2015-06-29
|
* win: compile with -debugGravatar Enrico Tassi2015-06-29
|
* Code documentation of the TACTIC/VERNAC EXTEND macros.Gravatar Pierre-Marie Pédrot2015-06-29
|
* Fix incompleteness of conversion used by evarconvGravatar Matthieu Sozeau2015-06-28
| | | | | | In case we need to backtrack on universe inconsistencies when converting two (incompatible) instances of the same constant and unfold them. Bug reported by Amin Timany.
* Reinstall Set Printing Universes option overwritten by Maxime!Gravatar Matthieu Sozeau2015-06-28
|
* Share prop/set values in sorts.ml.Gravatar Matthieu Sozeau2015-06-26
|
* Fix bug #4254 with the help of J.H. JourdanGravatar Matthieu Sozeau2015-06-26
| | | | | | | | | | | | | | | 1) We now _assign_ the smallest possible arities to mutual inductive types and eventually add leq constraints on the user given arities. Remove useless limitation on instantiating algebraic universe variables with their least upper bound if they have upper constraints as well. 2) Do not remove non-recursive variables when computing minimal levels of inductives. 3) Avoid modifying user-given arities if not necessary to compute the minimal level of an inductive. 4) We correctly solve the recursive equations taking into account the user-declared level.
* BUGFIX: Three fixes for the price of 1 in sorts.ml:Gravatar Matthieu Sozeau2015-06-26
| | | | | - Proper [family] implementation - Use the tailor made hash function for Sorts.t in two places.
* Add target to install dev files.Gravatar Matthieu Sozeau2015-06-26
|
* Introduction of a "Undelimit Scope" command, undoing "Delimit Scope"Gravatar Lionel Rieg2015-06-26
|
* Typos in my previous edition of the reference manual.Gravatar Assia Mahboubi2015-06-26
|
* Some edition in the coq_makefile/_CoqProject section.Gravatar Assia Mahboubi2015-06-26
| | | | | | There are still two items I do not undertand fully (the last one about -extra-phony, and the removal of external libraries at make clean time, that I could not reproduce on a toy example.
* Added _CoqProject to the index of the reference manual.Gravatar Assia Mahboubi2015-06-26
|
* Adding a more efficient representation of OCaml objects in votour.Gravatar Pierre-Marie Pédrot2015-06-25
|