aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FMapFacts.v
diff options
context:
space:
mode:
authorGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-09-04 09:43:36 +0000
committerGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-09-04 09:43:36 +0000
commit39f6bc84e726a6e3e09644b5b7e38c3c3475972b (patch)
treeb369b36917b4887acb7657db5aec556ead4c9f03 /theories/FSets/FMapFacts.v
parent9ef3acbdccba1733ba1543e700936d29290bad63 (diff)
Correction du bug #1937
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11359 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FMapFacts.v')
-rw-r--r--theories/FSets/FMapFacts.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/FSets/FMapFacts.v b/theories/FSets/FMapFacts.v
index 20f4623f9..e7dba21bd 100644
--- a/theories/FSets/FMapFacts.v
+++ b/theories/FSets/FMapFacts.v
@@ -975,7 +975,7 @@ Module WProperties (E:DecidableType)(M:WSfun E).
fold (fun k e b => if f k e then true else b) m false.
Definition partition (f : key -> elt -> bool)(m : t elt) :=
- (filter f m, filter (fun k e => negb (f k e))).
+ (filter f m, filter (fun k e => negb (f k e)) m).
Section Specs.
Variable f : key -> elt -> bool.