aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-24 20:48:15 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-24 20:48:15 +0000
commit72add906154ce22894a41cf04543a7c096456e09 (patch)
tree5dd21c4198789c6791b845008120c71b2058c95e /theories/QArith
parent2337b9bfc662981a2630df8c173d54b32fa2b2b6 (diff)
Tauto breaking not only binary "conjunctions" seems like a bad idea
after all... git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11259 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/QArith')
-rw-r--r--theories/QArith/Qreduction.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/QArith/Qreduction.v b/theories/QArith/Qreduction.v
index f289b6106..6b16cfff4 100644
--- a/theories/QArith/Qreduction.v
+++ b/theories/QArith/Qreduction.v
@@ -49,7 +49,7 @@ Proof.
Open Scope Z_scope.
intuition.
rewrite <- H in H0,H1; clear H.
- rewrite H5; rewrite H6.
+ rewrite H3; rewrite H4.
assert (0 <> g).
intro; subst g; discriminate.
@@ -57,7 +57,7 @@ Proof.
apply Zmult_gt_0_lt_0_reg_r with g.
omega.
rewrite Zmult_comm.
- rewrite <- H6; compute; auto.
+ rewrite <- H4; compute; auto.
rewrite Z2P_correct; auto.
ring.
Close Scope Z_scope.