aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
...
* Init: some results in Type should rather be Defined than QedGravatar letouzey2011-03-21
* Makefile.build: states/initial.coq was wrongly done with -dont-load-proofsGravatar letouzey2011-03-21
* Makefile.build: compile the stdlib with -dont-load-proofs by defaultGravatar letouzey2011-03-18
* A tatical "timeout <n> <tac>" that fails if <tac> hasn't finished in <n> secondsGravatar letouzey2011-03-18
* An option "Set Default Timeout n."Gravatar letouzey2011-03-17
* Goptions: repair Unset for int optionsGravatar letouzey2011-03-17
* CompareSpec: a slight generalization/reformulation of CompSpecGravatar letouzey2011-03-17
* Adapt printers.mllib after my last commitGravatar letouzey2011-03-16
* Finish branching functions handling module errors (cf. r13886)Gravatar letouzey2011-03-16
* Remove some weird syntax "fun ... ," that used to be accepted (cf r13876)Gravatar letouzey2011-03-16
* Adapt test-suite/output/Extraction_matchs_2413 to new indentation of extractionGravatar letouzey2011-03-16
* Fix inductive_template building ill-typed evars, and update test-suite scriptsGravatar msozeau2011-03-13
* - Add modulo_delta_types flag for unification to allow fullGravatar msozeau2011-03-13
* Keep information on which fields are subclasses in class declarations,Gravatar msozeau2011-03-11
* Inference of match predicate produces ill-typed unification problem,Gravatar msozeau2011-03-11
* Tentative to make unification check types at every instanciation of anGravatar msozeau2011-03-11
* - Better error messages taking unif. constraints into account.Gravatar msozeau2011-03-11
* Forgot a use of evars_reset_evd in nf_evars, add an optional argument asGravatar msozeau2011-03-10
* Do not forget conv_pbs when resetting an evm: Gravatar msozeau2011-03-10
* ZBits,ZdivEucl,ZDivFloor: a few lemmas with weaker preconditionsGravatar letouzey2011-03-10
* Solve evar instantiations in the right environment.Gravatar msozeau2011-03-08
* Fix declarations of [Add Setoid/Morphism...] in sections to not exportGravatar msozeau2011-03-08
* syntax for exponentsGravatar pottier2011-03-08
* adding eta in the vmGravatar bgregoir2011-03-08
* Reverted commit r13893 about propagation of more informativeGravatar herbelin2011-03-07
* Revert commit r13883: instantiating ?n by a lambda when "?n a" has toGravatar herbelin2011-03-07
* Added propagation of evars unification failure reasons for betterGravatar herbelin2011-03-07
* CHANGES: mentionning quickly Separate ExtractionGravatar letouzey2011-03-07
* Extraction: a warning when an opaque constant is enterredGravatar letouzey2011-03-07
* Extraction: fix printing of haskell modular namesGravatar letouzey2011-03-07
* Extraction: avoid printing unused mutual fix components (fix #2477)Gravatar letouzey2011-03-07
* A new command "Separate Extraction"Gravatar letouzey2011-03-07
* Added a table for using reserved names for binding names to typesGravatar herbelin2011-03-05
* Moving printing of module typing errors upwards to himsg.ml so as toGravatar herbelin2011-03-05
* Starting being more explicit on the reasons why module subtyping fails.Gravatar herbelin2011-03-05
* A few more betaiota on environments and types of error messages. Seems toGravatar herbelin2011-03-05
* Added support for instantiation of ?n by a lambda when "?n a" has toGravatar herbelin2011-03-05
* Reorganized a bit evarconv.ml:Gravatar herbelin2011-03-05
* Improved define_evar_as_lambda which was creating an unrelated new evarGravatar herbelin2011-03-05
* Instantiate evar by a lambda when "?n args" has to unify with ProdGravatar herbelin2011-03-05
* Fixed a "feature" about subtyping records: one was expected not onlyGravatar herbelin2011-03-05
* Restore documentation of library String which was removed in 2007 (r10049)Gravatar herbelin2011-03-05
* Forgotten removal of ',' in 'fun' rule: it has to come with the lambda notationGravatar herbelin2011-03-05
* Fixing injection bug #2493 (regression introduced by fixing injectionGravatar herbelin2011-03-05
* CHANGES: update of syntax for annotations of functor applicationGravatar letouzey2011-03-04
* Extraction: improved indentation of extracted code (fix #2497)Gravatar letouzey2011-03-04
* Simplify proofs in Permutation using generalized rewriting.Gravatar msozeau2011-03-04
* - Allow to set a particular transparent_state for the local hintGravatar msozeau2011-03-04
* checker: cleanupGravatar glondu2011-03-04
* checker: add eta-expansionGravatar glondu2011-03-04