aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Classes
Commit message (Expand)AuthorAge
...
* Delete trailing whitespaces in all *.{v,ml*} filesGravatar glondu2009-09-17
* Fix compilation errors due to last commit.Gravatar msozeau2009-09-15
* Stop using [obligation_tactic] from Program.Tactics as the defaultGravatar msozeau2009-09-15
* Misc fixes:Gravatar msozeau2009-09-10
* Fix the bug-ridden code used to choose leibniz or generalizedGravatar msozeau2009-09-08
* Do a fixpoint on the result of typeclass search to force theGravatar msozeau2009-06-08
* Stop using a "Manual Implicit Arguments" flag and support them as soonGravatar msozeau2009-05-27
* Minor fixes in typeclasses:Gravatar msozeau2009-05-16
* Improvements in typeclasses eauto and generalized rewriting:Gravatar msozeau2009-05-05
* Fixes for bugs in r12110:Gravatar msozeau2009-04-28
* - Implementation of a new typeclasses eauto procedure based on successGravatar msozeau2009-04-27
* Backporting 12080 (fixing bug #2091 on bad rollback in the "where"Gravatar herbelin2009-04-24
* Rename [Morphism] into [Proper] and [respect] into [proper] to complyGravatar msozeau2009-04-21
* Fix wrong pattern in Morphisms. Fix bug scripts to reflect the fact thatGravatar msozeau2009-04-20
* Just export RelationClasses for [Equivalence] through Setoid.Gravatar msozeau2009-04-18
* Only export the notations of Morphism as well as Equivalence throughGravatar msozeau2009-04-17
* Better Requires in Classes. Fix bug #2093: the code does not requireGravatar msozeau2009-04-16
* Rewrite of setoid_rewrite to modularize it based on proof-producingGravatar msozeau2009-04-13
* Move setoid_rewrite to its own module and do some clean up inGravatar msozeau2009-04-07
* Rewrite of Program Fixpoint to overcome the previous limitations: Gravatar msozeau2009-03-28
* Fix [subrelation] clauses that privileged the weakest. Better impl argsGravatar msozeau2009-02-04
* Last changes in type class syntax: Gravatar msozeau2009-01-18
* Move FunctionalExtensionality to Logic/ (someone please check that theGravatar msozeau2008-12-16
* Finish fix for the treatment of [inverse] in [setoid_rewrite], making aGravatar msozeau2008-12-16
* Generalized binding syntax overhaul: only two new binders: `() and `{},Gravatar msozeau2008-12-14
* Fix handling of [inverse] in setoid_rewrite, with an hopefully completeGravatar msozeau2008-12-08
* Fix priority of the Leibniz Setoid instance to 10 (thanks to M. LassonGravatar msozeau2008-12-04
* More factorization of inductive/record and typeclasses: move classGravatar msozeau2008-11-09
* Minor fixes:Gravatar msozeau2008-11-05
* Fix bug #1977 by allowing the [apply] variants to take an [open_constr]Gravatar msozeau2008-10-23
* Generalized implementation of generalization.Gravatar msozeau2008-10-23
* Add user syntax for creating hint databases [Create HintDb fooGravatar msozeau2008-09-14
* Use manual implicts in Classes and rationalize class parameter names.Gravatar msozeau2008-09-14
* Remove redefinition of id in Program.Basics, just add maximal implicits.Gravatar msozeau2008-09-13
* Add enough information to correctly globalize recursive calls in inductive andGravatar msozeau2008-09-11
* Add the ability to declare [Hint Extern]'s with no pattern.Gravatar msozeau2008-09-07
* Improve typeclasses eauto using the dnet for local assumptions too, and selectGravatar msozeau2008-09-04
* Fix bug #1935, reworking the reflexivity, symmetry... tactics to useGravatar msozeau2008-09-03
* Major speed and space improvements in setoid rewrite:Gravatar msozeau2008-08-27
* Fix dependency problem that makes compilation fail :)Gravatar msozeau2008-08-23
* - New auto hints for transparency/opacity control, not bound to Gravatar msozeau2008-08-22
* Fixes in dependent induction tactic to keep names, allow givingGravatar msozeau2008-08-21
* Even better test for choosing rewrite or setoid_rewrite.Gravatar msozeau2008-07-26
* More compatibility fixes, revert the tauto fix that preventedGravatar msozeau2008-07-25
* New tactics [conv] to test convertibility (actually, unification) of twoGravatar msozeau2008-07-22
* - Improve [Context] vernacular to allow arbitrary binders, not justGravatar msozeau2008-07-07
* Fixes in handling of implicit arguments:Gravatar msozeau2008-07-04
* Various bug fixes in type classes and subtac:Gravatar msozeau2008-07-01
* Enhanced discrimination nets implementation, which can now work withGravatar msozeau2008-06-27
* Rename obligations_tactic to obligation_tactic and fix bugs #1893.Gravatar msozeau2008-06-22