diff options
Diffstat (limited to 'theories/Classes/Init.v')
-rw-r--r-- | theories/Classes/Init.v | 16 |
1 files changed, 10 insertions, 6 deletions
diff --git a/theories/Classes/Init.v b/theories/Classes/Init.v index 762cc5c1..f6e51018 100644 --- a/theories/Classes/Init.v +++ b/theories/Classes/Init.v @@ -6,22 +6,26 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(* Initialization code for typeclasses, setting up the default tactic +(** * Initialization code for typeclasses, setting up the default tactic for instance search. Author: Matthieu Sozeau - Institution: LRI, CNRS UMR 8623 - UniversitĂcopyright Paris Sud - 91405 Orsay, France *) + Institution: LRI, CNRS UMR 8623 - University Paris Sud +*) -(* $Id: Init.v 12187 2009-06-13 19:36:59Z msozeau $ *) +(* $Id$ *) (** Hints for the proof search: these combinators should be considered rigid. *) Require Import Coq.Program.Basics. -Typeclasses Opaque id const flip compose arrow impl iff. +Typeclasses Opaque id const flip compose arrow impl iff not all. -(** The unconvertible typeclass, to test that two objects of the same type are +(** Apply using the same opacity information as typeclass proof search. *) + +Ltac class_apply c := autoapply c using typeclass_instances. + +(** The unconvertible typeclass, to test that two objects of the same type are actually different. *) Class Unconvertible (A : Type) (a b : A) := unconvertible : unit. |