aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FMapPositive.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-21 13:03:16 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-21 13:03:16 +0000
commit1d874af4b89c3c13551ce3648924b1b7ee6fcc24 (patch)
tree4efa6ffc523ad9d5d9b2d96a38c59cd92644ca55 /theories/FSets/FMapPositive.v
parent0a235f0d6ed807600ccf5534af7ed6f8657d1274 (diff)
incomplete and temporary fix for PR#1222: revert accepts up to 10 args
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9156 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FMapPositive.v')
-rw-r--r--theories/FSets/FMapPositive.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/FSets/FMapPositive.v b/theories/FSets/FMapPositive.v
index 7c6374899..9008b3623 100644
--- a/theories/FSets/FMapPositive.v
+++ b/theories/FSets/FMapPositive.v
@@ -734,7 +734,7 @@ Module PositiveMap <: S with Module E:=PositiveOrderedTypeBits.
Proof.
intros.
generalize (xelements_complete _ _ _ _ H); clear H; intros.
- revert H; revert v; revert m; revert q; revert p0.
+ revert p0 q m v H.
induction p; destruct p0; simpl; intros; eauto; try discriminate.
Qed.
@@ -743,7 +743,7 @@ Module PositiveMap <: S with Module E:=PositiveOrderedTypeBits.
Proof.
intros.
generalize (xelements_complete _ _ _ _ H); clear H; intros.
- revert H; revert v; revert m; revert q; revert p0.
+ revert p0 q m v H.
induction p; destruct p0; simpl; intros; eauto; try discriminate.
Qed.