aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* Deprecate options -dont, -lazy, -force-load-proofs.Gravatar Guillaume Melquiond2014-06-13
| | | | | | | These options no longer have any impact on the way proofs are loaded. In other words, loading is always lazy, whatever the options. Keeping them just so that coqc dies when the user prints some opaque symbol does not seem worth it.
* Less ocaml warnings.Gravatar Hugo Herbelin2014-06-13
|
* Improving tclWITHHOLES which did not see undefined evars up toGravatar Hugo Herbelin2014-06-13
| | | | | restriction, after last fix commit which precisely possibly restricts evars of a term "t" in "apply t in H" without resolving them.
* Fixing "clear" in internal_cut_replace: forbid dependencies in theGravatar Hugo Herbelin2014-06-13
| | | | name of replaced hypothesis.
* Improved error message when a meta posed as an evar remains unsolvedGravatar Hugo Herbelin2014-06-13
| | | | in case prefix 'e' of "apply" and co is not given.
* Check resolution of Metas turned into Evars by pose_all_metas_as_evarsGravatar Hugo Herbelin2014-06-13
| | | | in unification.ml in case prefix 'e' of "apply" and co is not given.
* Fixing wrong environment for Meta's in pose_all_metas_as_evars (bug #3284).Gravatar Hugo Herbelin2014-06-13
|
* Adapt simpl/cbn unfolding and refolding machinery to projections, so thatGravatar Matthieu Sozeau2014-06-13
| | | | primitive projections obey the Arguments command.
* Code cleaning in Univ.Gravatar Pierre-Marie Pédrot2014-06-12
|
* Passing some tactics to the new monad type.Gravatar Pierre-Marie Pédrot2014-06-12
|
* Fix bug #3291, stack overflow in rewrite.Gravatar Matthieu Sozeau2014-06-11
|
* Fix bug #3289Gravatar Matthieu Sozeau2014-06-11
|
* Move bug # 3368 to closed bugsGravatar Matthieu Sozeau2014-06-11
|
* Merge branch 'more-test-suite' of https://github.com/JasonGross/coq into trunkGravatar Matthieu Sozeau2014-06-11
|\
* | - Fix bug #3368, due to wrong use of the Cst_stack for projections.Gravatar Matthieu Sozeau2014-06-11
| | | | | | | | | | - Monomorphize Cst_stack to 'a = constr. - Add corresponding debug printer.
* | In generalized rewrite, avoid retyping completely and constantly the ↵Gravatar Matthieu Sozeau2014-06-11
| | | | | | | | | | | | | | conclusion, and results of unifying the lemma with subterms. Using Retyping.get_type_of instead results in 3x speedup in Ncring_polynom.
* | fix handling of side effects in abstract (fixes QArithSternBrocot)Gravatar Enrico Tassi2014-06-11
| | | | | | | | | | The right fix should probably be to remove the build_constant_by_tactic function and only use the build_by_tactic one
| * Add many more cases to the test-suiteGravatar Jason Gross2014-06-10
| | | | | | | | | | | | | | | | | | I'd add more, but I'm tired and it's late and I should sleep. Maybe I'll pick up at 3279 (working down) another day. Bug 3344 is broken; [Fail Defined.] says that [Defined] has not failed, even though it raises an anomaly. So there's no way I can think of to test it. I've left it in the [opened] directory anyway.
| * Move closed bug 3314Gravatar Jason Gross2014-06-10
| |
| * Add a test-case for bug #3314 proving FalseGravatar Jason Gross2014-06-10
|/
* Fixing Sorting Universes in a world where le and lt constraints may beGravatar Pierre-Marie Pédrot2014-06-10
| | | | redundant in canonical arcs.
* Compute the trace of a universe inconsistency only when explicitly requiredGravatar Pierre-Marie Pédrot2014-06-10
| | | | by the printing options (i.e. when "Print Universes" is set).
* Made explanations for universe inconsistencies optional. They are only usedGravatar Pierre-Marie Pédrot2014-06-10
| | | | by the printer anyway.
* Specialize the type of [Univ.compare_neq] so that it is clear it is only usedGravatar Pierre-Marie Pédrot2014-06-10
| | | | to recover the trace of a universe inconsistency. Changed its name too btw.
* Removing dead code in checker/univ.ml.Gravatar Pierre-Marie Pédrot2014-06-10
|
* Removing explanations of universe inconsistencies from the checker. TheyGravatar Pierre-Marie Pédrot2014-06-10
| | | | were never used and were responsible for code duplication.
* Imperatively check touched universes in compare_neq functions. This ensuresGravatar Pierre-Marie Pédrot2014-06-10
| | | | | | a O(1) check, contrasting with the previous O(n) behaviour that rendered universe constraint checking prohibitive on big files. I expect a 20% speedup on such files.
* Providing the checker with its own version of the Univ file.Gravatar Pierre-Marie Pédrot2014-06-10
| | | | | I also took the opportunity to remove a lot of code not used by the checker.
* - Fix substitution of universes which needlessly hashconsed existing universes.Gravatar Matthieu Sozeau2014-06-10
| | | | - More cleanup. remove unneeded functions in universes
* Oops, one refactoring was not compiled.Gravatar Matthieu Sozeau2014-06-10
|
* More cleanup/reorganizing of univ.ml to separate constraint/universe ↵Gravatar Matthieu Sozeau2014-06-10
| | | | | | handling from the instance/contexts and substitution code.
* Fix module order in printers.mllibGravatar Matthieu Sozeau2014-06-10
|
* Cleanup in Univ, moving code for UniverseConstraints outside the kernel in ↵Gravatar Matthieu Sozeau2014-06-10
| | | | | | | | Universes. Needed to exponse compare_head_gen(_leq) so that it could be reused in Universes. Remove unused functions from univ as well and refactor a little bit. Changed the syntax to Type@{} for explicit universe level specs, following the WG decision.
* Remove unused function in univGravatar Matthieu Sozeau2014-06-10
|
* Merge branch 'hott-test-suite-progress' of https://github.com/JasonGross/coq ↵Gravatar Matthieu Sozeau2014-06-10
|\ | | | | | | into trunk
* | Flattening Level module structure in Univ.Gravatar Pierre-Marie Pédrot2014-06-09
| |
| * Mark some progress in the HoTT/coq test-suiteGravatar Jason Gross2014-06-08
| | | | | | | | | | | | I've marked new failing commands that I'm confused about with "???"; I'm not sure whether or not they should fail there, but we should keep the test-suite compiling, probably.
* | Adding a toplevel option allowing to deactivate the term sharing in kernelGravatar Pierre-Marie Pédrot2014-06-08
|/ | | | reduction.
* Moving hook code from Future to Lemmas. This seemed to disrupt compilation ofGravatar Pierre-Marie Pédrot2014-06-08
| | | | the checker, and it was not used before that anyway.
* Fix canonical structure resolution in unification (bug found in Ssreflect).Gravatar Matthieu Sozeau2014-06-08
|
* Timeout implementation for Windows based on threads.Gravatar Pierre-Marie Pédrot2014-06-08
|
* Enforce a correct exception handling in declaration_hooksGravatar Enrico Tassi2014-06-08
| | | | | | | This should finally get rid of the following class of bugs: Qed fails, STM undoes to the beginning of the proof because the exception is not annotated with the correct state, PG gets out of sync because errors always refer to the last command in PGIP.
* ind_tables: always declare side effects (Closes: HOTT#110)Gravatar Enrico Tassi2014-06-08
| | | | | | | | | | | | | | | | | | | | | | | | declare takes care of ignoring side effects that are available in the global environment. This is yet another instance of what the "abominion" (aka abstract) can do: the code was checking for the existence in the environment of the elimination principle, and not regenerating it (nor declaring the corresponding side effect) if the elimination principle is used twice. Of course to functionalize the imperative actions on the environment when two proofs generated by abstract use the same elim principle, such elim principle has to be inlined twice, once in each abstracted proof. In other words, a side effect generated by a tactic inside an abstract is *global* but will be made local, si it must always be declared, no matter what. Now the system works like this: - side effects are always declared, even if a caching mechanism thinks the constant is already there (it can be there, no need to regenerate it but the intent to generate it *must* be declared anyhow) - at Qed time, we filter the list of side effects and decide which ones are really needed to be inlined. bottom line: STOP using abstract.
* STM: handle "Time Abort" correctly (Closes: 3332)Gravatar Enrico Tassi2014-06-08
|
* Function in Univ uselessly exported.Gravatar Pierre-Marie Pédrot2014-06-08
|
* Removing 'open Univ' from checker.Gravatar Pierre-Marie Pédrot2014-06-07
|
* Moving a Thread.yield in check_interrupt.Gravatar Pierre-Marie Pédrot2014-06-07
|
* Adding a new Control file centralizing the control options of Coq.Gravatar Pierre-Marie Pédrot2014-06-07
|
* Preserve compatibility on examples such as "intros []." on goals suchGravatar Hugo Herbelin2014-06-06
| | | | | | | as "forall x:nat*nat, x=x", which resulted in "forall n n0 : nat, (n, n0) = (n, n0)" before commit 37f68259ab0a33c3b5b41de70b08422d9bcd3bec on "Fixing introduction patterns * and ** ".
* Dead code.Gravatar Hugo Herbelin2014-06-06
|