aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* Changing syntax "$(tactic)$" into "ltac:(tactic)", as discussed in WG.Gravatar Hugo Herbelin2015-12-02
|
* Univs/Program: update the universe context with global universeGravatar Matthieu Sozeau2015-12-02
| | | | | constraints at the time of Next Obligation/Solve Obligations so that interleaving definitions and obligation solving commands works properly.
* Fix bug #4444: Next Obligation performed after a Section opening wasGravatar Matthieu Sozeau2015-12-02
| | | | | | | using the wrong context. This is very bad style but currently unavoidable, at least we don't throw an anomaly anymore.
* Add an option to deactivate compatibility printing of primitiveGravatar Matthieu Sozeau2015-12-02
| | | | projections (off by default).
* Fix a bug in externalisation which prevented printing of projectionsGravatar Matthieu Sozeau2015-12-02
| | | | using dot notation.
* vio: fix argument parsing (progress on #4442)Gravatar Enrico Tassi2015-12-01
|
* Test for bug #4149.Gravatar Pierre-Marie Pédrot2015-11-30
|
* Test-suite files for closed bugsGravatar Matthieu Sozeau2015-11-28
|
* Closed bugs.Gravatar Matthieu Sozeau2015-11-28
|
* Univs: correctly register universe binders for lemmas.Gravatar Matthieu Sozeau2015-11-28
|
* Univs: entirely disallow instantiation of polymorphic constants withGravatar Matthieu Sozeau2015-11-27
| | | | | | | | | Prop levels. As they are typed assuming all variables are >= Set now, and this was breaking an invariant in typing. Only one instance in the standard library was used in Hurkens, which can be avoided easily. This also avoids displaying unnecessary >= Set constraints everywhere.
* Avoid recording spurious Set <= Top.i constraints which are alwaysGravatar Matthieu Sozeau2015-11-27
| | | | valid (when Top.i is global and hence > Set).
* Fix [Polymorphic Hint Rewrite].Gravatar Matthieu Sozeau2015-11-27
|
* Fixing the "parsing rules with idents later declared as keywords" problem.Gravatar Hugo Herbelin2015-11-26
| | | | | | | The fix was actually elementary. The lexer comes with a function to compare parsed tokens against tokens of the parsing rules. It is enough to have this function considering an ident in a parsing rule to be equal to the corresponding string parsed as a keyword.
* Make the pretty printer resilient to incomplete nametab (progress on #4363).Gravatar Enrico Tassi2015-11-26
| | | | | | | | | | | | | | The nametab in which the error message is printed is not the one in which the error message happens. This reveals a weakness in the fix_exn code: the fix_exn function should be pure, while in some cases (like this one) uses the global state (the nametab) to print a term in a pretty way (the shortest non-ambiguous name for constants). This patch makes the externalization phase (used by term printing) resilient to an incomplete nametab, so that printing a term in the wrong nametab does not mask the original error.
* Adding the Printing Projections options to the index.Gravatar Pierre-Marie Pédrot2015-11-26
|
* Fix for case-insensitive path looking continued (#2554): Adding aGravatar Hugo Herbelin2015-11-25
| | | | | second chance to dynamically regenerate the file system cache when a file is not found (suggested by Guillaume M.).
* Generalizing the patch to bug #2554 on fixing path looking withGravatar Hugo Herbelin2015-11-25
| | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | | correct case on MacOS X whose file system is case-insensitive but case-preserving (HFS+ configured in case-insensitive mode). Generalized it to any case-preserving case-insensitive file system, which makes it applicable to Windows with NTFS used in case-insensitive mode but also to Linux when mounting a case-insensitive file system. Removed the blow-up of the patch, improved the core of the patch by checking whether the case is correct only for the suffix part of the file to be found (not for the part which corresponds to the path in which where to look), and finally used a cache so that the effect of the patch is not observable. Note that the cache is implemented in a way not synchronous with backtracking what implies e.g. that a file compiled in the middle of an interactive session would not be found until Coq is restarted, even by backtracking before the corresponding Require. For history see commits b712864e9cf499f1298c1aca1ad8a8b17e145079, 4b5af0d6e9ec1343a2c3ff9f856a019fa93c3606 69941d4e195650bf59285b897c14d6287defea0f e7043eec55085f4101bfb126d8829de6f6086c5a. as well as https://coq.inria.fr/bugs/show_bug.cgi?id=2554 discussion on coq-club "8.5 and MathClasses" (May 2015) discussion on coqdev "Coq awfully slow on MacOS X" (Sep 2015)
* Heuristic to check the version of lablgtk2 in configure.ml.Gravatar Pierre-Marie Pédrot2015-11-25
| | | | | When not using ocamlfind, we use a grep-based heuristic to check that lablgtk2 is recent enough. This is an extension of an already-used heuristic.
* Reverting 1467c225 (Fixing an old typo in Retyping, found by Matej).Gravatar Hugo Herbelin2015-11-25
| | | | This was not a typo (was correctly taking the family type of the type).
* Advertising that CoqIDE requires lablgtk >= 2.16Gravatar Pierre-Marie Pédrot2015-11-25
|
* Checking lablgtk version in configure. Fix bug #4423.Gravatar Pierre-Marie Pédrot2015-11-25
|
* Univs: carry on universe substitution when defining obligations ofGravatar Matthieu Sozeau2015-11-24
| | | | | non-polymorphic definitions, original universes might be substituted later on due to constraints.
* Fixing an old typo in Retyping, found by Matej.Gravatar Hugo Herbelin2015-11-24
|
* Fix generation of equality schemes on polymorphic equality types.Gravatar Matthieu Sozeau2015-11-23
|
* Fix output of universe arcs. (Fix bug #4422)Gravatar Guillaume Melquiond2015-11-23
|
* Fixing a vm_compute bug in the presence of let-ins among theGravatar Hugo Herbelin2015-11-22
| | | | parameters of an inductive type.
* Fixing a bug of adjust_subst_to_rel_context.Gravatar Hugo Herbelin2015-11-22
|
* Fixing kernel bug in typing match with let-ins in the arity.Gravatar Hugo Herbelin2015-11-22
| | | | | | | | | | Was exploitable in 8.3, 8.4 and 8.5beta1. A priori not exploitable in 8.5beta2 and 8.5beta3 from a Coq file because typing done while compiling "match" would serve as a protection. However exploitable by calling the kernel directly, e.g. from a plugin (but a plugin can anyway do what it wants by bypassing kernel type abstraction). Fixing similar error in pretyping.
* Univs: generation of induction schemes should not generated uselessGravatar Matthieu Sozeau2015-11-20
| | | | | | instances for each of the inductive in the same block but reuse the original universe context shared by all of them. Also do not force schemes to become universe polymorphic.
* Univs: fix type_of_global_in_context not returning instantiated universe ↵Gravatar Matthieu Sozeau2015-11-20
| | | | contexts.
* Fix bug #4429: eauto with arith: 70x performance regression in Coq 8.5.Gravatar Pierre-Marie Pédrot2015-11-19
| | | | | | | | | | | The issue was due to the fact that unfold hints are given a priority of 4 by default. As eauto was now using hint priority rather than the number of goals produced to order the application of hints, unfold were almost always used too late. We fixed this by manually giving them a priority of 1 in the eauto tactic. Also fixed the relative order of proof depth w.r.t. hint priority. It should not be observable except for breadth-first search, which is seldom used.
* Allow program hooks to see the refined universe_context at the end of aGravatar Matthieu Sozeau2015-11-19
| | | | | definition, if they manipulate structures depending on the initial state of the context.
* Fix bug #4433, removing hack on evars appearing in a pattern from aGravatar Matthieu Sozeau2015-11-19
| | | | | constr, and the associated signature, not needed anymore. Update CHANGES, no evar_map is produced by pattern_of_constr anymore.
* Fixing fix c71aa6b to primitive projections.Gravatar Hugo Herbelin2015-11-18
| | | | | | | | | | | | - Introduced an error: fold was counting in the wrong direction and I did not test it. Sorry. - Substitution from params-with-let to params-without-let was still not correct. Hopefully everything ok now. Eventually, we should use canonical combinators for that: extended_rel_context to built the instance and and a combinator apparently yet to define for building a substitution contracting the let-ins.
* Fix a bug preventing the generation of graphs when doing multipleGravatar Matthieu Sozeau2015-11-18
| | | | pattern-matching on function calls.
* Improve error message.Gravatar Maxime Dénès2015-11-18
|
* MacOS package script: do not fail if link to /Applications already exists.Gravatar Maxime Dénès2015-11-18
|
* Slightly documenting code for building primitive projections.Gravatar Hugo Herbelin2015-11-18
|
* Fixing logical bugs in the presence of let-ins in computiong primitiveGravatar Hugo Herbelin2015-11-18
| | | | | | | | | projections. - lift accounting for the record missing in computing the subst from fields to projections of the record - substitution for parameters should not lift the local definitions - typo in building the latter (subst -> letsubst)
* More optimizations of [Clenv.clenv_fchain].Gravatar Pierre-Marie Pédrot2015-11-17
| | | | | Everywhere we know that the universes of the left argument are an extension of the right argument, we do not have to merge universes.
* Performance fix for destruct.Gravatar Pierre-Marie Pédrot2015-11-17
| | | | | | The clenv_fchain function was needlessly merging universes coming from two evarmaps even though one was an extension of the other. A flag was added so that the tactic just retrieves the newer universes.
* Being more precise and faithful about the origin of the file reportingGravatar Hugo Herbelin2015-11-16
| | | | about the prehistory of Coq.
* Continue fix of PMP, handling setoid_rewrite in let-bound hyps correctly.Gravatar Matthieu Sozeau2015-11-13
|
* MacOS package script: do not fail if directory _dmg already exists.Gravatar Maxime Dénès2015-11-13
|
* Fix bug #4412: [rewrite] (setoid_rewrite?) creates ill-typed terms.Gravatar Pierre-Marie Pédrot2015-11-12
| | | | | We retypecheck the hypotheses introduced by the refine primitive instead of blindly trusting them when the unsafe flag is set to false.
* Fixed test-suite file for bug #3998.Gravatar Matthieu Sozeau2015-11-12
|
* Update CHANGESGravatar Jason Gross2015-11-12
| | | | Mention compatibility file.
* Script building MacOS package.Gravatar Maxime Dénès2015-11-12
|
* Now closed.Gravatar Matthieu Sozeau2015-11-11
|