aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar Raphaël Monat <raphael.monat@ens-lyon.org>2017-10-27 10:46:41 +0200
committerGravatar Raphaël Monat <raphael.monat@ens-lyon.org>2017-10-27 10:46:41 +0200
commit84e274fb6d36bbd8306c2977520ebe1cf410349a (patch)
treef49bb16803a262303d2d10e6784f626d6df2f7dc /theories
parent5431b0f17cd73a09472093e779cc1508b3b3ac4f (diff)
Chaining two tactics in a proof
Diffstat (limited to 'theories')
-rw-r--r--theories/QArith/QArith_base.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/QArith/QArith_base.v b/theories/QArith/QArith_base.v
index 66740512b..5996d30f2 100644
--- a/theories/QArith/QArith_base.v
+++ b/theories/QArith/QArith_base.v
@@ -188,7 +188,7 @@ Qed.
Lemma Qeq_bool_trans x y z: Qeq_bool x y = true -> Qeq_bool y z = true -> Qeq_bool x z = true.
Proof.
- rewrite !Qeq_bool_iff. apply Qeq_trans.
+ rewrite !Qeq_bool_iff; apply Qeq_trans.
Qed.
Hint Resolve Qnot_eq_sym : qarith.