aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith/Qreduction.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/QArith/Qreduction.v')
-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 6b16cfff4..f289b6106 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 H3; rewrite H4.
+ rewrite H5; rewrite H6.
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 <- H4; compute; auto.
+ rewrite <- H6; compute; auto.
rewrite Z2P_correct; auto.
ring.
Close Scope Z_scope.