aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FSetEqProperties.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-01-28 05:08:18 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-01-28 05:08:18 +0000
commit47e9afaaa4c08aca97d4f4b5a89cb40da76bd850 (patch)
treea2424086c8b7e1635f7a481109a7fae8fcaad386 /theories/FSets/FSetEqProperties.v
parent3f6196a6bdc7e5b0e6d8279a7b7b0de74faa3492 (diff)
Tentative to fix bug #2628 by not letting intuition break records. Might be too much of a backwards-incompatible change
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14949 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/FSets/FSetEqProperties.v')
-rw-r--r--theories/FSets/FSetEqProperties.v2
1 files changed, 0 insertions, 2 deletions
diff --git a/theories/FSets/FSetEqProperties.v b/theories/FSets/FSetEqProperties.v
index 755bc7dd0..3a2de94b5 100644
--- a/theories/FSets/FSetEqProperties.v
+++ b/theories/FSets/FSetEqProperties.v
@@ -920,8 +920,6 @@ Lemma sum_compat :
forall s, (forall x, In x s -> f x=g x) -> sum f s=sum g s.
intros.
unfold sum; apply (fold_compat _ (@Logic.eq nat)); auto with *.
-intros x x' Hx y y' Hy. rewrite Hx, Hy; auto.
-intros x x' Hx y y' Hy. rewrite Hx, Hy; auto.
Qed.
End Sum.