aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FSetFacts.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-06-11 16:34:28 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-06-11 16:34:28 +0000
commitfcdfc18ee51940460daa68e241c0951438276ddd (patch)
tree6a750d898b75fe664a21caed349ffd2603b50a42 /theories/FSets/FSetFacts.v
parent5caebcd8ff2bedae02a23d79251a2344c7aea4d6 (diff)
undeletion of E_ST and Equal_ST: these records aren't mandatory, but quite useful
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9887 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FSetFacts.v')
-rw-r--r--theories/FSets/FSetFacts.v10
1 files changed, 10 insertions, 0 deletions
diff --git a/theories/FSets/FSetFacts.v b/theories/FSets/FSetFacts.v
index 4c1c51c49..ac0227f5c 100644
--- a/theories/FSets/FSetFacts.v
+++ b/theories/FSets/FSetFacts.v
@@ -287,6 +287,16 @@ End BoolSpec.
(** * [E.eq] and [Equal] are setoid equalities *)
+Definition E_ST : Setoid_Theory elt E.eq.
+Proof.
+constructor; [apply E.eq_refl|apply E.eq_sym|apply E.eq_trans].
+Qed.
+
+Definition Equal_ST : Setoid_Theory t Equal.
+Proof.
+constructor; [apply eq_refl | apply eq_sym | apply eq_trans].
+Qed.
+
Add Relation elt E.eq
reflexivity proved by E.eq_refl
symmetry proved by E.eq_sym