aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FMapWeakList.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-04-29 11:57:59 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-04-29 11:57:59 +0000
commitc03302b1783ddd7a78902689b57787bed67c1f88 (patch)
tree23d7a4959eb05f7d7de6f29d360d54f8fff6a64c /theories/FSets/FMapWeakList.v
parent91e2e89e84c0eb343198b0c887b727b35f9658cd (diff)
meilleur nommage pour PairOrderedType
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8772 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FMapWeakList.v')
-rw-r--r--theories/FSets/FMapWeakList.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/FSets/FMapWeakList.v b/theories/FSets/FMapWeakList.v
index f2a324aca..bfa97d0b2 100644
--- a/theories/FSets/FMapWeakList.v
+++ b/theories/FSets/FMapWeakList.v
@@ -24,7 +24,7 @@ Arguments Scope list [type_scope].
Module Raw (X:DecidableType).
-Module PX := PairDecidableType X.
+Module PX := KeyDecidableType X.
Import PX.
Definition key := X.t.
@@ -34,7 +34,7 @@ Section Elt.
Variable elt : Set.
-(* now in PairDecidableType:
+(* now in KeyDecidableType:
Definition eqk (p p':key*elt) := X.eq (fst p) (fst p').
Definition eqke (p p':key*elt) :=
X.eq (fst p) (fst p') /\ (snd p) = (snd p').