aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins
Commit message (Expand)AuthorAge
* In Coq_config: get rid of coqsrc and make coqlib optionalGravatar glondu2011-09-27
* Added support for referring to subterms of the goal by pattern.Gravatar herbelin2011-09-26
* Generalizing subst_term_occ so that it supports an arbitrary matchingGravatar herbelin2011-09-26
* Fix commit 14489: missing Coq. in dirpathGravatar letouzey2011-09-23
* Program: add some check_required_library (fix #2592) + some dead code removalGravatar letouzey2011-09-23
* Omega: for non-arithmetical goals, try proving False from context (wish #2236)Gravatar letouzey2011-09-16
* Omega aware of Z.pred (fix #1912)Gravatar letouzey2011-09-15
* correction du bug 2047Gravatar jforest2011-09-09
* Improved ltac code for zify (fix #2575).Gravatar letouzey2011-09-06
* Extraction Implicit: fix the numbering of constructor argumentsGravatar letouzey2011-09-05
* Bug 2589: Documentation patch of Hendrik TewsGravatar pboutill2011-09-02
* Extraction: allow extraction of records with anonymous fields (fix #2555)Gravatar letouzey2011-08-25
* New proposition "rewrite Heq in H" for eq_rect (assuming that there isGravatar herbelin2011-08-08
* Esubst: make types of substitutions & lifts privateGravatar puech2011-08-08
* moins de reification inutile, noatations standardsGravatar pottier2011-08-04
* 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
* 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
* Extraction: replace generic = on mutual_inductive_body by mib_equalGravatar 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
* Nsatz: replaced some generic = on constr by eq_constrGravatar puech2011-07-29
* Recdef: replaced some generic = on constr by eq_constrGravatar puech2011-07-29
* FourierR: replaced some generic Hashtbl on constr by ConstrhashGravatar puech2011-07-29
* Refl_omega: replaced generic = on constr by eq_constrGravatar puech2011-07-29
* Newring: replaced some generic = on constr by eq_constrGravatar puech2011-07-29
* Refl_omega: replaced some generic = on constr by eq_constrGravatar puech2011-07-29
* Const_omega: replaced some generic = on constr by eq_constrGravatar puech2011-07-29
* Functional_principles_types: replaced some generic = on constr by eq_constrGravatar puech2011-07-29
* Newring: replaced generic = on constr by eq_constrGravatar puech2011-07-29
* Coq_omega: replaced generic = on constr by eq_constrGravatar puech2011-07-29
* Quote: replaced generic = on constr by eq_constrGravatar puech2011-07-29
* Coq_omega: replaced many generic = on constr by eq_constrGravatar puech2011-07-29
* Newring: generic Pervasives.compare on constr replaced by constr_ordGravatar puech2011-07-29
* Term: moved function constr_ord (a.k.a compare_constr) from Sequent to TermGravatar puech2011-07-29
* Ccalgo, Ccproof: multiple generic Hashtbl on constr and term replaced by Cons...Gravatar puech2011-07-29
* Newring: generic equality on constr replaced by constr_equalGravatar puech2011-07-29
* Ccproof: generic equality on term replaced by term_equalGravatar puech2011-07-29
* Sequent: generic equality on global_reference replaced by RefOrdered.compareGravatar puech2011-07-29
* Sequent: generic equality on kernel_name replaced by kn_ordGravatar puech2011-07-29
* Sequent: generic equality on constr replaced by destructorsGravatar puech2011-07-29
* Sequent: generic equality on ident replaced by id_ordGravatar puech2011-07-29
* Instances: generic equality on global_reference replaced by RefOrdered.compareGravatar puech2011-07-29
* Unify: generic equality on constr replaced by eq_constrGravatar puech2011-07-29
* Integral domainsGravatar pottier2011-07-26
* Ring2 devient Ncring et la reification par les type classes est partageeGravatar pottier2011-07-26