From 84e274fb6d36bbd8306c2977520ebe1cf410349a Mon Sep 17 00:00:00 2001 From: Raphaƫl Monat Date: Fri, 27 Oct 2017 10:46:41 +0200 Subject: Chaining two tactics in a proof --- theories/QArith/QArith_base.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/QArith') 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. -- cgit v1.2.3