aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures/OrdersTac.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-13 16:53:01 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-13 16:53:01 +0000
commite0e008cef9f5b2ead64708651f52b739a8225993 (patch)
treec78fd9c28394c52f347baeed39ba91a4a3f6a812 /theories/Structures/OrdersTac.v
parent4fdec1dc05525f1c5f9b52566b6dcfd02bf3c219 (diff)
Try to avoid re-declaring Equivalence, especially for Logic.eq
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12662 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Structures/OrdersTac.v')
-rw-r--r--theories/Structures/OrdersTac.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/theories/Structures/OrdersTac.v b/theories/Structures/OrdersTac.v
index 80be89026..35484ae77 100644
--- a/theories/Structures/OrdersTac.v
+++ b/theories/Structures/OrdersTac.v
@@ -304,7 +304,8 @@ Definition lt := flip O.lt.
Definition le := flip O.le.
Include EqLtLeNotation.
-Instance eq_equiv : Equivalence eq.
+(* No Instance syntax to avoid saturating the Equivalence tables *)
+Definition eq_equiv := O.eq_equiv.
Instance lt_strorder: StrictOrder lt.
Proof. unfold lt; auto with *. Qed.