aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Collapse)AuthorAge
* Tests for bugs #3509 and #3510.Gravatar Pierre-Marie Pédrot2015-07-28
|
* Fixing bug #3509 and #3510 (anomalies in "tactics/term_dnet.ml").Gravatar Pierre-Marie Pédrot2015-07-28
| | | | | | Commit dc438047 was a bit overlooked as it introduced a wrong comparison function on term patterns in dnets. Strangely enough, it seems not to have wreaked havoc that much compared to the severity of the error.
* Use open_utf8_file_in for opening files in the IDE. (Fix bug #2874)Gravatar Guillaume Melquiond2015-07-28
| | | | | | | | File system.ml seemed like a better choice than util.ml for sharing the code, but it was bringing a bunch of useless dependencies to the IDE. There are presumably several other tools that would benefit from using open_utf8_file_in instead of open_in, e.g. coqdoc.
* Test for bug #2243.Gravatar Pierre-Marie Pédrot2015-07-27
|
* Fixing #4305 (compatibility wrt 8.4 in not interpreting anGravatar Hugo Herbelin2015-07-27
| | | | | | | abbreviation not bound to an applied constructor as itself but rather as a binding variable as it was the case for non-applied constructor). This was broken by e5c02503 while fixed #3483 (Not_found uncaught with a notation to a non-constructor).
* Slightly improving line break formatting in Info command.Gravatar Hugo Herbelin2015-07-27
|
* Improving over 26aa224293 in reporting unexpected error during scheme creation.Gravatar Hugo Herbelin2015-07-27
| | | | | This should actually probably be an anomaly, but I'm unsure the code for decidability schemes is robust enough to dare it.
* Fixing bug #3736 (anomaly instead of error/warning/silence onGravatar Hugo Herbelin2015-07-27
| | | | | | | | | | | | | | decidability scheme). Not clear to me why it is not a warning (in verbose mode) rather than silence when a scheme supposed to be built automatically cannot be built, as in: Set Decidable Equality Schemes. Inductive a := A with b := B. which could explain why a_beq and a_eq_dec as well as b_beq and b_eq_dec are not built.
* Output test for bug #2169.Gravatar Pierre-Marie Pédrot2015-07-27
|
* Fixing bug #2169:Gravatar Pierre-Marie Pédrot2015-07-27
| | | | "Print Module command shows module type expression incorrectly".
* Regenerate the axiom figure of the FAQ.Gravatar Guillaume Melquiond2015-07-26
| | | | | | The .png was ugly (less than 400px wide) and did not match the content of the .fig file (e.g. presence of '$'). To improve things a bit, text is now rendered by latex.
* Remove obsolete question about eta-conversion.Gravatar Guillaume Melquiond2015-07-26
|
* Using maps and sets instead of lists in coqdep.Gravatar Pierre-Marie Pédrot2015-07-24
| | | | | | The quadratic behaviour of list searching probably appears with small enough samples. With the advent of usable libraries in Coq, and thus many possible dependencies, better be safe than sorry.
* Fixing bug #4265: "coqdep does not handle From ... Require" for good.Gravatar Pierre-Marie Pédrot2015-07-24
|
* Silence `which`Gravatar Jason Gross2015-07-23
| | | | On Fedora, `which 2>&1 >/dev/null` doesn't silence stderr, while `which >/dev/null 2>&1` does.
* adding a missing case for printing zippers.Gravatar Gregory Malecha2015-07-23
|
* a small amount of documentation on the virtual machine.Gravatar Gregory Malecha2015-07-23
|
* Removing the G_xml module again.Gravatar Pierre-Marie Pédrot2015-07-22
| | | | | The file seems to have been reintroduced by error by commit 012fe1a96, but it was not compiled anyway.
* Refman: document Show Universes.Gravatar Matthieu Sozeau2015-07-22
|
* test-suite: add test for bug# 3743.Gravatar Matthieu Sozeau2015-07-22
|
* Extraction: fix primitive projection extraction.Gravatar Matthieu Sozeau2015-07-22
| | | | Use expand projection to come back to the projection-as-constant encoding, dealing with parameters correctly.
* Fix incomplete pattern-matching.Gravatar Matthieu Sozeau2015-07-22
| | | | | I was not seeing the warning due to the 10 deprecation warnings before it...
* Remove obsolete documentation. (Fix bug #4238)Gravatar Guillaume Melquiond2015-07-22
|
* Fixing bug #4303: Anomaly: Uncaught exception Invalid_argument.Gravatar Pierre-Marie Pédrot2015-07-21
|
* Refining 71def2f8 on too strong occur-check limiting evar-evarGravatar Hugo Herbelin2015-07-16
| | | | | | | | | | | | unification in tactics. The relaxing of occur-check was ok but was leading trivial problems of the form ?X[?Meta] = ?X[?Meta] to enter a complex Evar-ization into ?X[?Meta] = ?X[?Y], ?Meta:=?Y which consider_remaining_unif_problems was not any more able to deal with. Doing quick: treat the trivial cases ?X[args] = ?X[args] in an ad hoc way, so that it behaves as if the occur-check had not been restricted.
* Slight improvement in naming anonymous variables in error messages:Gravatar Hugo Herbelin2015-07-16
| | | | | | | | | | | | | | | | | | using closer naming strategies for naming variables in make_all_name_different and when contracting trivial letins. Not sure what the best policy is. Maybe the contraction process should not invent names at al and let make_all_name_different do the job. Maybe pretyping should name all rels which it pushes to environment (with cases.ml paying attention to avoid clash). The problem shows for instance with a PretypeError (... env, ... , ActualTypeNotCoercible (NotClean (... env ...)) message with two copies of env which we don't if they are the same but which have to share same names for similar rendering of the rels! This was revealed e.g. by the error message of #4177.
* Fixing #4177 (find_projectable was liable to ask to instantiate an evar twice).Gravatar Hugo Herbelin2015-07-16
| | | | This is a bug in a pretty old code, showing also in 8.3 and 8.4.
* Remove old test file for #3819 (now fixed).Gravatar Maxime Dénès2015-07-16
|
* Fixing bug #4240 (closure_of_filter was not ensuring refinement ofGravatar Hugo Herbelin2015-07-16
| | | | | former filter after 48509b61 and 3cd718c, because filtered let-ins were not any longer preserved).
* Test file for #3819.Gravatar Maxime Dénès2015-07-16
|
* Fix universe instantiation with canonical structures.Gravatar Maxime Dénès2015-07-16
| | | | | | | Patch by Matthieu Sozeau. Fixes #3819: "Error: Unsatisfied constraints" due to canonical structure inference
* Modules: fix bug #4294Gravatar Matthieu Sozeau2015-07-16
| | | | | We were throwing away constraints from 'with Definition' in module type ascriptions.
* Continuing 93579407, spotting other potential sources of anomalyGravatar Hugo Herbelin2015-07-16
| | | | | because of the name of a bound variable lost when unifying under a binder in evarconv.
* Fixing anomaly #3743 while printing an error message involving evar constraints.Gravatar Hugo Herbelin2015-07-16
| | | | | | | | Indeed, the name of a bound variable was lost when unifying under a Prod in evarconv. The error message for "Unable to satisfy the following constraints" is still to be improved though.
* Univs/Inductive: fix typechecking of casesGravatar Matthieu Sozeau2015-07-15
| | | | | | | I was trying to be a bit too clever with not substituting the universe instance everywhere: the constructor type/inductive arity has to be instantiated before instantiate_params runs, which became true only for constructor types since my last commit.
* STM: fix a "exn with no safe id attached" error on a failing queryGravatar Enrico Tassi2015-07-14
| | | | It showed up at the CoqCS.
* Updating checksum in checker (9c732a5cc continued).Gravatar Hugo Herbelin2015-07-12
| | | | | | Calling md5sum test earlier, at the time coqchk is built, rather than at testing time, hopefully moving it closer to what it is supposed to occur.
* CoqIDE: recenter on backtrack (Close: #4277)Gravatar Enrico Tassi2015-07-11
|
* Rewording about how to upgrade on failing calls to constructor.Gravatar Hugo Herbelin2015-07-10
|
* Unused variables reported by OCaml.Gravatar Hugo Herbelin2015-07-10
|
* Continuing handling of NoCoercion after df6e64fd28 and 4944b5e72.Gravatar Hugo Herbelin2015-07-10
| | | | | | | | | | Commit df6e64fd28 let apply_coercion raise NoCoercion untrapped by inh_app_fun. Commit 4944b5e72 caught NoCoercion but missed re-attempting inserting a coercion after resolving instances of type classes. This fixes MathClasses (while preserving fix of part of from 4944b5e72 and fixes of HoTT_coq_014.v from df6e64fd28).
* Option -type-in-type: added support in checker and making it contaminatingGravatar Hugo Herbelin2015-07-10
| | | | | | | | | | in vo files (this was not done yet in 24d0027f0 and 090fffa57b). Reused field "engagement" to carry information about both impredicativity of set and type in type. For the record: maybe some further checks to do around the sort of the inductive types in coqchk?
* Highlighting Universe in CoqIDE.Gravatar Hugo Herbelin2015-07-10
|
* CHANGES: grammatical correction, suggested by Jason Gross on Bugzilla.Gravatar Maxime Dénès2015-07-10
|
* Native compiler: make non-fatal linking errors silent except in debug mode.Gravatar Maxime Dénès2015-07-10
|
* 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.