aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Classes/Equivalence.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-09-14 18:23:59 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-09-14 18:23:59 +0000
commita49d5036279440e6c35e54eda05f425696aba8ca (patch)
tree218d86fc456e0dd40f01e868d8fd34b4ea114f22 /theories/Classes/Equivalence.v
parent3c8057d3c28b9243328ecb1f0a8197b11cf9fd77 (diff)
Add user syntax for creating hint databases [Create HintDb foo
[discriminated]] with a switch for using the more experimantal dnet impl for every hint. Also add [Hint Transparent/Opaque] which parameterize the dnet and the unification flags used by auto/eauto with a particular database. Document all this. Remove [Typeclasses unfold] directives that are no longer needed (everything is unfoldable by default) and move to [Typeclasses Transparent/Opaque] syntax. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11409 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Classes/Equivalence.v')
-rw-r--r--theories/Classes/Equivalence.v4
1 files changed, 0 insertions, 4 deletions
diff --git a/theories/Classes/Equivalence.v b/theories/Classes/Equivalence.v
index 9909f18ad..ef85c14aa 100644
--- a/theories/Classes/Equivalence.v
+++ b/theories/Classes/Equivalence.v
@@ -29,8 +29,6 @@ Open Local Scope signature_scope.
Definition equiv [ Equivalence A R ] : relation A := R.
-Typeclasses unfold equiv.
-
(** Overloaded notations for setoid equivalence and inequivalence. Not to be confused with [eq] and [=]. *)
Notation " x === y " := (equiv x y) (at level 70, no associativity) : equiv_scope.
@@ -43,8 +41,6 @@ Open Local Scope equiv_scope.
Definition pequiv [ PER A R ] : relation A := R.
-Typeclasses unfold pequiv.
-
(** Overloaded notation for partial equivalence. *)
Infix "=~=" := pequiv (at level 70, no associativity) : equiv_scope.