aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith/QArith_base.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/QArith/QArith_base.v')
-rw-r--r--theories/QArith/QArith_base.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/theories/QArith/QArith_base.v b/theories/QArith/QArith_base.v
index 121527c63..66740512b 100644
--- a/theories/QArith/QArith_base.v
+++ b/theories/QArith/QArith_base.v
@@ -176,19 +176,19 @@ Proof.
apply eq_true_iff_eq. rewrite !Qeq_bool_iff. now symmetry.
Qed.
-Lemma Qeq_bool_refl x: is_true (Qeq_bool x x).
+Lemma Qeq_bool_refl x: Qeq_bool x x = true.
Proof.
- unfold is_true. rewrite Qeq_bool_iff. now reflexivity.
+ rewrite Qeq_bool_iff. now reflexivity.
Qed.
-Lemma Qeq_bool_sym x y: is_true (Qeq_bool x y) -> is_true (Qeq_bool y x).
+Lemma Qeq_bool_sym x y: Qeq_bool x y = true -> Qeq_bool y x = true.
Proof.
- unfold is_true. rewrite !Qeq_bool_iff. now symmetry.
+ rewrite !Qeq_bool_iff. now symmetry.
Qed.
-Lemma Qeq_bool_trans x y z: is_true (Qeq_bool x y) -> is_true (Qeq_bool y z) -> is_true (Qeq_bool x z).
+Lemma Qeq_bool_trans x y z: Qeq_bool x y = true -> Qeq_bool y z = true -> Qeq_bool x z = true.
Proof.
- unfold is_true. rewrite !Qeq_bool_iff. apply Qeq_trans.
+ rewrite !Qeq_bool_iff. apply Qeq_trans.
Qed.
Hint Resolve Qnot_eq_sym : qarith.