aboutsummaryrefslogtreecommitdiffhomepage
Commit message (Expand)AuthorAge
* OrderedType2 : trivial lemmas are turned into tests for order.Gravatar letouzey2009-10-16
* Structure/OrderTac.v : highlight the "order" tactic by isolating it from FSet...Gravatar letouzey2009-10-16
* note for later : when the tag table is shared, never, ever create twoGravatar vgross2009-10-16
* typo in doc of Extraction BlacklistGravatar letouzey2009-10-15
* MSetInterface: (W)Raw2Sets splitted in 2 (helps a future commit by Elie)Gravatar letouzey2009-10-15
* OrderedType2.order is slightly weaker since last commit, adapt accordinglyGravatar letouzey2009-10-15
* OrderedType2.order : fix the last fix (a fail at the wrong place)Gravatar letouzey2009-10-15
* Fix bug in typeclass resolution discoverd by Eeelis van der Weegen:Gravatar msozeau2009-10-15
* Typo in last commitGravatar letouzey2009-10-14
* Improved tactic "order" in OrderedTypeGravatar letouzey2009-10-14
* Made implicit arguments of Operators_Properties.v localGravatar herbelin2009-10-13
* Typos.Gravatar gmelquio2009-10-13
* Better handling of emphasis.Gravatar msozeau2009-10-13
* MSets: a new generation of FSetsGravatar letouzey2009-10-13
* Fix bug #2162 and a name clashing bug in generalized binders.Gravatar msozeau2009-10-09
* Fix a typo(?) in previous commitGravatar letouzey2009-10-09
* Fixed clash names in Relations (see bug report #2152) and make namesGravatar herbelin2009-10-08
* Init/Tactics.v: tactic with nicer name 'exfalso' for 'elimtype False'Gravatar letouzey2009-10-08
* Implicit argument of Logic.eq become maximally insertedGravatar letouzey2009-10-08
* Fixed a bug introduced in revision 12265.Gravatar herbelin2009-10-08
* Fix for missing hypotesae in XML proof tree export.Gravatar cek2009-10-07
* Fixed installation of Coqide interface/library files (bug #2147).Gravatar gmelquio2009-10-06
* Relaxed error severity when encountering unknown library objects or tacticGravatar gmelquio2009-10-06
* Correctly do backtracking during type class resolution even if only newGravatar msozeau2009-10-05
* Revert "kills the old backtracking framework and replaces it with"Gravatar vgross2009-10-05
* Changed the way to support compatibility with previous versions.Gravatar herbelin2009-10-04
* Removal of trailing spaces.Gravatar serpyc2009-10-04
* Some new lemmas on max and min and a fix for a wrongly stated lemma in r12358.Gravatar herbelin2009-10-04
* Fixed small name freshness bug in Functional Scheme ("Heq" name wasGravatar herbelin2009-10-03
* A few additions in Min.v.Gravatar herbelin2009-10-03
* Added option "Unset Dependent Propositions Elimination" to protectGravatar herbelin2009-10-03
* Add support for Local Declare ML ModuleGravatar glondu2009-09-29
* Remove legacy export_* functionsGravatar glondu2009-09-29
* kills the old backtracking framework and replaces it withGravatar vgross2009-09-29
* Fix the stdlib doc compilation + switch all .v file to utf8Gravatar letouzey2009-09-28
* Applied patches from BSD/pkgsrc maintainer, so that Coq compiles out-of-the-box.Gravatar gmelquio2009-09-28
* Apply "Declare Implicit Tactic" also to terms interpreted as "openGravatar herbelin2009-09-27
* Fixed a bug in the interaction between dEqThen and inject_at_positionsGravatar herbelin2009-09-27
* Fixed two tests that was incorrectly typed in former revisions 12348 and 12356.Gravatar herbelin2009-09-27
* Add a few properties about Rmin/Rmax with replication in Zmin/Zmax.Gravatar herbelin2009-09-27
* Fixed error message "cannot infer the type of id" in presence ofGravatar herbelin2009-09-27
* Delay the choice of eliminator in destruct/induction until we know ifGravatar herbelin2009-09-27
* Complement to 12347 and 12348 on the extended syntax of case/elim.Gravatar herbelin2009-09-27
* Fixed a hole in glob_tactic that allowed some Ltac code to refer toGravatar herbelin2009-09-26
* Micromega doc : psatz Z -> psatz Z 2Gravatar fbesson2009-09-24
* Ltac doc: only variables are accepted as message_tokenGravatar glondu2009-09-23
* Add the option to automatically introduce variables declared before theGravatar msozeau2009-09-22
* Better use of transparency information for local hypotheses: Gravatar msozeau2009-09-22
* Update link to "Recursive Make Considered Harmful"Gravatar glondu2009-09-21
* Only one "in" clause in "destruct" even for a multiple "destruct".Gravatar herbelin2009-09-20