| Commit message (Expand) | Author | Age |
... | |
* | Change Hint Resolve, Immediate to take a global reference as argument | msozeau | 2012-10-26 |
* | Removing redundant definition of case_eq (see #2919). | herbelin | 2012-10-16 |
* | Updating headers. | herbelin | 2012-08-08 |
* | Legacy Ring and Legacy Field migrated to contribs | letouzey | 2012-07-05 |
* | Some cleanup in recent proofs concerning pi | letouzey | 2012-07-05 |
* | Kills the useless tactic annotations "in |- *" | letouzey | 2012-07-05 |
* | Open Local Scope ---> Local Open Scope, same with Notation and alii | letouzey | 2012-07-05 |
* | ZArith + other : favor the use of modern names instead of compat notations | letouzey | 2012-07-05 |
* | These files are displaced from Rtrigo.v and Ranalysis_reg.v | bertot | 2012-06-11 |
* | finish the rearrangement for removing the sin_PI2 axiom. This new version | bertot | 2012-06-11 |
* | Adds the proof of PI_ineq, plus some other smarter ways to approximate PI | bertot | 2012-06-11 |
* | Modifications and rearrangements to remove the action that sin (PI/2) = 1 | bertot | 2012-06-05 |
* | Fixing tauto "special" behavior on singleton types w/ 2 parameters (bug #2680). | herbelin | 2012-04-15 |
* | theories/, plugins/ and test-suite/ ported to the Arguments vernacular | gareuselesinge | 2011-11-21 |
* | Cleaning a little bit the files talking about descriptions: avoiding | herbelin | 2011-11-03 |
* | BinInt: Z.add become the alternative Z.add' | letouzey | 2011-05-05 |
* | - Improve unification (beta-reduction, and same heuristic as evarconv for red... | msozeau | 2011-04-13 |
* | Fix scripts relying on unification not doing any beta reduction. | msozeau | 2011-04-13 |
* | Unify meta types with the right flags, add betaiotazeta reduction to unificat... | msozeau | 2011-04-13 |
* | CompareSpec: a slight generalization/reformulation of CompSpec | letouzey | 2011-03-17 |
* | Remove the "Boxed" syntaxes and the const_entry_boxed field | letouzey | 2011-01-28 |
* | First release of Vector library. | pboutill | 2010-12-10 |
* | Some more revision of {P,N,Z}Arith + bitwise ops in Ndigits | letouzey | 2010-11-18 |
* | Solve name conflict about pow introduced by commit 13546. | letouzey | 2010-10-21 |
* | Numbers: new functions pow, even, odd + many reorganisations | letouzey | 2010-10-14 |
* | Updated all headers for 8.3 and trunk | herbelin | 2010-07-24 |
* | 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 |
* | 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 |
* | Removed Rlimit's dependency on Classical. | gmelquio | 2010-02-17 |
* | Removed Rderiv's dependency on Classical. | gmelquio | 2010-02-17 |
* | Nicer names: DecidableType2* --> Equalities*, OrderedType2* --> Orders* | letouzey | 2010-01-07 |
* | Rework of GenericMinMax: new axiomatic, split logical/decidable parts, Leibni... | letouzey | 2010-01-07 |
* | OrderTac: use TotalOrder, no more "change" before calling "order" (stuff with... | letouzey | 2010-01-07 |
* | Reverse order of arguments in min_case_strong for better uniformity (and comp... | letouzey | 2009-12-17 |
* | Factorisation between Makefile and ocamlbuild systems : .vo to compile are in... | letouzey | 2009-12-09 |
* | Fix anomaly when using typeclass resolution with filtered hyps in evars. | msozeau | 2009-12-06 |
* | Taking advantage of the new "Include Self Type" in DecidableType2 and NZAxioms | letouzey | 2009-11-16 |
* | DecidableType: A specification via boolean equality as an alternative to eq_dec | letouzey | 2009-11-10 |
* | ROrderedType + Rminmax : Coq's Reals can be seen as OrderedType. | letouzey | 2009-11-03 |
* | Remove various useless {struct} annotations | letouzey | 2009-11-02 |
* | Added alternate versions of existing lemmas on sqrt. | gmelquio | 2009-11-02 |
* | Init/Tactics.v: tactic with nicer name 'exfalso' for 'elimtype False' | letouzey | 2009-10-08 |
* | Removal of trailing spaces. | serpyc | 2009-10-04 |
* | Some new lemmas on max and min and a fix for a wrongly stated lemma in r12358. | herbelin | 2009-10-04 |
* | Fix the stdlib doc compilation + switch all .v file to utf8 | letouzey | 2009-09-28 |
* | Add a few properties about Rmin/Rmax with replication in Zmin/Zmax. | herbelin | 2009-09-27 |