aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
* New fix for is_ident_not_keyword.Gravatar herbelin2011-08-13
* Fixes mini-bug: Qed would succeed even on focused proofs.Gravatar aspiwack2011-08-12
* SearchAbout and similar: add a customizable blacklistGravatar letouzey2011-08-11
* Propagated information from the reduction tactics to the kernel soGravatar herbelin2011-08-10
* Fixing typos in commentsGravatar herbelin2011-08-10
* Improving error message about coinductive guard (old "cases" is now "match")Gravatar herbelin2011-08-10
* Fixing printing bug with last trailing non-maximally implicitGravatar herbelin2011-08-10
* Exported tactic intro_thenGravatar herbelin2011-08-10
* Made CHANGES more uniformly writtenGravatar herbelin2011-08-10
* Take benefit of bullets available by default in PreludeGravatar herbelin2011-08-10
* Less ambitious application of a notation for eq_rect. We proposedGravatar herbelin2011-08-10
* Partly revert commit r14389 about relaxing the condition for being a keywordGravatar herbelin2011-08-10
* Fix implementation of Hint Immediate used by typeclasses eautoGravatar msozeau2011-08-10
* Added list_map_filter_iGravatar msozeau2011-08-10
* Graceful error message for [Proof Mode] and [Set Default Proof Mode] when req...Gravatar aspiwack2011-08-10
* BinInt: more structured scripts thanks to bullets and { }Gravatar letouzey2011-08-09
* Coqide: revised parsing of coq sentencesGravatar letouzey2011-08-09
* In coqtop, a terminating "." must now be followed by a blank or eof.Gravatar letouzey2011-08-09
* Moved the declaration of "Classic" being the default proof mode to coqtop.ml ...Gravatar aspiwack2011-08-09
* Some forgotten lemma in Arith with "O" in the name instead of "0".Gravatar herbelin2011-08-08
* New proposition "rewrite Heq in H" for eq_rect (assuming that there isGravatar herbelin2011-08-08
* Be a bit less aggressive in declaring idents as keywords in notationsGravatar herbelin2011-08-08
* Two bugs in pattern-matching compilation:Gravatar herbelin2011-08-08
* Term: fix hash_constr to hash modulo casts & names (like compare_constr)Gravatar puech2011-08-08
* Esubst: make types of substitutions & lifts privateGravatar puech2011-08-08
* moins de reification inutile, noatations standardsGravatar pottier2011-08-04
* Fix unification: detect invalid evar instantiations due to scoping earlier.Gravatar msozeau2011-08-04
* Fix nf_evars_undefined use in pr_constraintsGravatar msozeau2011-08-03
* Fix nf_evars_undefinedGravatar msozeau2011-08-03
* Patch to simplify is_open_canonical_projectionGravatar herbelin2011-08-02
* More robust evar_map debugging printerGravatar herbelin2011-08-02
* Term: simplify compare_constr by removing calls to decompose_appGravatar puech2011-08-01
* Added .dir-locals file to take advantage of emacs 23's new Directory-local va...Gravatar puech2011-08-01
* fixed bug 2580. Quick fix: copy emitcodes before patching itGravatar barras2011-08-01
* Ring: replaced various generic = on constr by eq_constr, destructors etc.Gravatar puech2011-07-29
* Quote: replaced various generic = on constr by eq_constr, destructors etc.Gravatar puech2011-07-29
* generic = on named_context replaced by named_context_equalGravatar puech2011-07-29
* Newring: generic = on constr replaced by eq_constrGravatar puech2011-07-29
* Coq_micromega: generic = on constr replaced by eq_constrGravatar puech2011-07-29
* Field: generic Gmap on constr replaced by CmapGravatar puech2011-07-29
* Extract_env: generic = on prec_declaration replaced by prec_declaration_equalGravatar puech2011-07-29
* Tactics: replace generic = on constr by destructorsGravatar puech2011-07-29
* Auto: replace generic compare on pri_auto_tactic by pri_auto_tactic_ordGravatar puech2011-07-29
* Extraction: replace generic = on mutual_inductive_body by mib_equalGravatar puech2011-07-29
* Evarutil: replace generic list_distinct on constr by constr_list_distinctGravatar puech2011-07-29
* replaced some generic = on constr by eq_constrGravatar puech2011-07-29
* Subtac_cases: replaced some generic = on constr by destructorsGravatar puech2011-07-29
* Ring: replaced some generic Pervasives.compare on constr by constr_ordGravatar puech2011-07-29
* Add printer dependency to Hashtbl_alt (used in Term)Gravatar puech2011-07-29
* Nsatz: replaced some generic = on constr by eq_constrGravatar puech2011-07-29