aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
...
* Added Add LoadPath in coqdep lexer (but not in coqdep itself by lack of time).Gravatar herbelin2011-10-29
* Fixed broken globalization of identifiers containing utf8 lettersGravatar herbelin2011-10-29
* Added checksums to glob files and warned about possibly missingGravatar herbelin2011-10-29
* Remove dynamic stuff from constr_expr and glob_constrGravatar glondu2011-10-28
* Remove avoidable use of GDynamicGravatar glondu2011-10-27
* Deactivating second-order pattern-matching in evarconv for 8.4.Gravatar herbelin2011-10-26
* Fix configuration box bug in recursive callGravatar pboutill2011-10-26
* Coq_makefile handles .mlpack filesGravatar pboutill2011-10-26
* Coqdep handles .mlpackGravatar pboutill2011-10-26
* Checker/subtyping.ml: avoid adding in env a module already there (fix #2609)Gravatar letouzey2011-10-26
* When checking for emptiness, use Foo.is_empty instead of (=) Foo.emptyGravatar letouzey2011-10-26
* Environ.set_universes is dead codeGravatar letouzey2011-10-26
* Mod_subst: some simplifications, some more significant names to functions, etcGravatar letouzey2011-10-26
* Auto: avoid storing clausenv (and hence env, evar_map, universes) in voGravatar letouzey2011-10-26
* Makefile install rule fixGravatar pboutill2011-10-26
* Coq_makefile includes coqtop -config without file generationGravatar pboutill2011-10-26
* Coq_makefile: libraries in bytecode are now installed tooGravatar pboutill2011-10-26
* Revision 14605 continued (Utf8.v now correctly exporting Utf8_core.v).Gravatar herbelin2011-10-26
* Applying Tom Prince's patch to support parametric "constructor n" inGravatar herbelin2011-10-25
* Merge common notations from Utf8.v and Utf8_core.v (see bug report #2610).Gravatar herbelin2011-10-25
* Regression tests for bugs #2613 and #2616.Gravatar herbelin2011-10-25
* First attempt at making Print Assumption compatible with opaque modules (fix ...Gravatar letouzey2011-10-25
* Coq_makefile: a more complete commentary about global variablesGravatar pboutill2011-10-25
* Coq_makefile does not install/compile explicitely cmo and cmxs? that are in a...Gravatar pboutill2011-10-25
* coqdep defines a makefile variable name_MLLIB_DEPENDENCIES to store dependenc...Gravatar pboutill2011-10-25
* Fixing use of type constraint for refining the "return" clause of "match".Gravatar herbelin2011-10-25
* Continuing r14585 (ill-typed restriction bug).Gravatar herbelin2011-10-25
* Fixing "destruct" test.Gravatar herbelin2011-10-25
* Continuing r1492 (useless changes were inadvertantly committed)Gravatar herbelin2011-10-25
* New strategy to infer return predicate of match construct whenGravatar herbelin2011-10-25
* Still more unification in typing.mlGravatar herbelin2011-10-25
* Icons in CoqIdE preference panelGravatar pboutill2011-10-25
* Configuration window of CoqIdE looks more like other Gtk one.Gravatar pboutill2011-10-25
* Heads: avoid potentially uncaught Not_found via an assert falseGravatar letouzey2011-10-24
* Mod_subst: Attempt to fix #2608Gravatar letouzey2011-10-24
* More unification in type_of and addition of e_type_of to get the newGravatar herbelin2011-10-24
* Fixing another bug revealing ill-typed use of evar restriction.Gravatar herbelin2011-10-24
* Fixing instance/filter mismatch in materialize_evar + documentation.Gravatar herbelin2011-10-24
* Fixing failing printer when the type of a binder name with implicitGravatar herbelin2011-10-24
* Fail if some conv pbs remain after consider_remaining_unif_problems.Gravatar herbelin2011-10-22
* Now consider remaining conversion problems in solve_remaining_evars.Gravatar herbelin2011-10-22
* Use also second-order unification if first-order fails at the time of conside...Gravatar herbelin2011-10-22
* Use full conversion for checking type of holes in destruct over aGravatar herbelin2011-10-22
* Fixing uncaught exception in pr_evar_map (pr_global failed for unknown global...Gravatar herbelin2011-10-22
* Fixing Equality.injectable which did not detect an equality withoutGravatar herbelin2011-10-22
* More descriptive error messages in checkerGravatar glondu2011-10-20
* Extraction.tex: typo in an Extract Inductive example (fix #2625)Gravatar letouzey2011-10-18
* Fix bug #2473 due to wrong folding of the evar environmentGravatar msozeau2011-10-18
* Fix bug #2227Gravatar msozeau2011-10-18
* Fix inductive coercion code in Program (bug #2378)Gravatar msozeau2011-10-18