| Commit message (Expand) | Author | Age |
* | Tentative fix for bug #2226: put inj_pair2 and eq_dep_eq hints in a | msozeau | 2010-06-09 |
* | Fixing commit r13090 (forgot to commit the file generating Nmake_gen.v). | herbelin | 2010-06-08 |
* | Made option "Automatic Introduction" active by default before too many | herbelin | 2010-06-08 |
* | Fix unfolding tactic for well-founded Programs. | msozeau | 2010-06-08 |
* | Ascii: simplier ascii_of_pos, conversion from/to N, proofs about nat-->ascii-... | letouzey | 2010-06-04 |
* | Correction program_simplify. Devrait corriger certaines contribs. | aspiwack | 2010-05-28 |
* | Generalized the formulation of classic_set in propositional contexts | herbelin | 2010-05-28 |
* | Added UIP_dec on suggestion of Eelis on #coq irc. | herbelin | 2010-05-22 |
* | Discontinue support for ocaml 3.09.* | letouzey | 2010-05-19 |
* | Added a few informations about file lineages (for the most part in kernel) | herbelin | 2010-05-09 |
* | Remove the svn-specific $Id$ annotations | letouzey | 2010-04-29 |
* | Here comes the commit, announced long ago, of the new tactic engine. | aspiwack | 2010-04-22 |
* | Compare_dec : a few better proofs (and extracted terms), some more Defined | letouzey | 2010-04-16 |
* | Granting wish #2229 (InA_dec transparent) and Michael Day's coq-club | herbelin | 2010-04-10 |
* | Change definition of FSetList so that equality is Leibniz | glondu | 2010-04-09 |
* | Small improvements around coqdoc (including fix for bug #2288) | herbelin | 2010-03-30 |
* | Fixing bug #2254 (inappropriate names of Zlt_gt_succ and Zlt_succ_gt) | herbelin | 2010-03-28 |
* | NMake: remove useless tactics abstract_pair, nicer comments | letouzey | 2010-03-10 |
* | NMake: Reorganization, interface for NMake_gen, explicit View, tactic destr_t... | letouzey | 2010-03-10 |
* | NMake_gen.ml: robustness w.r.t size, remove old commented stuff about shiftl | letouzey | 2010-03-10 |
* | Reorder resolution of type class and unification constraints. | msozeau | 2010-03-07 |
* | Minor fixes. | msozeau | 2010-03-05 |
* | Removed redundant and ill-named technical lemma. | gmelquio | 2010-02-18 |
* | Removed SeqProp's dependency on Classical. | gmelquio | 2010-02-18 |
* | Removed Rtrigo's dependency on Classical. | gmelquio | 2010-02-18 |
* | Removed Rseries' dependency on Classical. | gmelquio | 2010-02-17 |
* | RelationClasses: adapt eq_Reflexive and co to avoid Universe Inconsistencies | letouzey | 2010-02-17 |
* | Kill some useless dependencies (Bvector, Program.Syntax) | letouzey | 2010-02-17 |
* | Arith's min and max placed in Peano (+basic specs max_l and co) | letouzey | 2010-02-17 |
* | Removed Rlimit's dependency on Classical. | gmelquio | 2010-02-17 |
* | Removed Rderiv's dependency on Classical. | gmelquio | 2010-02-17 |
* | Uniformisation Sorting/Mergesort and Structures/Orders | letouzey | 2010-02-16 |
* | CompSpec2Type is used to build functions, it should be Defined, not Qed | letouzey | 2010-02-13 |
* | CompSpecType, a clone of CompSpec but in Type instead of Prop | letouzey | 2010-02-12 |
* | Cleanup in Classes, removing unsupported code. | msozeau | 2010-02-11 |
* | Min, Max: for avoiding inelegant NPeano.max printing, we Export this lib | letouzey | 2010-02-10 |
* | Euclidean division for NArith | letouzey | 2010-02-10 |
* | Fix [Existing Class] impl and add documentation. Fix computation of the | msozeau | 2010-02-10 |
* | Numbers: properties of min/max with respect to 0,S,P,add,sub,mul | letouzey | 2010-02-09 |
* | NPeano improved, subsumes NatOrderedType | letouzey | 2010-02-09 |
* | NSub: a missing lemma (sub usually decreases) | letouzey | 2010-02-09 |
* | NBinary improved, contains more, subsumes NOrderedType | letouzey | 2010-02-09 |
* | ZBinary (impl of Numbers via Z) reworked, comes earlier, subsumes ZOrderedType | letouzey | 2010-02-09 |
* | DoubleCyclic + NMake : typeclasses, more genericity, less ML macro-generation | letouzey | 2010-02-08 |
* | Update CHANGES, add documentation for new commands/tactics and do a bit | msozeau | 2010-01-30 |
* | Division in numbers: kills some Include to avoid bad alias Zsucc = ZDiv.Z.Z'.S | letouzey | 2010-01-29 |
* | Support for generalized rewriting under dependent binders, using the | msozeau | 2010-01-26 |
* | Add [Next Obligation with tactic] support (wish #1953). | msozeau | 2010-01-26 |
* | NMake (and hence BigN): shiftr, shiftl now in the signature NSig | letouzey | 2010-01-25 |
* | NMake: several things need not be macro-generated | letouzey | 2010-01-25 |