aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FSetDecide.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-06 17:00:52 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-06 17:00:52 +0000
commit0cdfa2fb137989f75cdebfa3a64726bc0d56a8af (patch)
treeaf9f649911bf82636fa24704ae095fc4247da94f /theories/FSets/FSetDecide.v
parent86b28df4c6029d43a0f12ab7c2d85cc13f4f60f1 (diff)
avoid duplicated creation of WFacts instances
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11064 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FSetDecide.v')
-rw-r--r--theories/FSets/FSetDecide.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/theories/FSets/FSetDecide.v b/theories/FSets/FSetDecide.v
index e8d639003..fe6623c33 100644
--- a/theories/FSets/FSetDecide.v
+++ b/theories/FSets/FSetDecide.v
@@ -22,6 +22,7 @@ Require Import Decidable DecidableTypeEx FSetFacts.
(** First, a version for Weak Sets *)
Module WDecide (E : DecidableType)(Import M : WSfun E).
+ Module F := FSetFacts.WFacts E M.
(** * Overview
This functor defines the tactic [fsetdec], which will
@@ -462,7 +463,7 @@ the above form:
the predicates [In] and [E.eq] applied only to
variables. We are going to use them with [autorewrite].
*)
- Module F := FSetFacts.WFacts E M.
+
Hint Rewrite
F.empty_iff F.singleton_iff F.add_iff F.remove_iff
F.union_iff F.inter_iff F.diff_iff