aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith
diff options
context:
space:
mode:
authorGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-08-17 13:43:52 +0000
committerGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-08-17 13:43:52 +0000
commitfbc1924f292b442d7c0dd565df83889f912f5477 (patch)
treee3269482f8a07b1a17ef1a82b7f5acef7a631b90 /theories/QArith
parentaf4283e8e4e670b8a5761892548f2d65792cd7e9 (diff)
Smaller proof terms for QcPower_{0,pos}
The use of compute produces huge terms that contain hundreds of unfolded Zadd, Zmul, Zsucc! git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14412 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/QArith')
-rw-r--r--theories/QArith/Qcanon.v8
1 files changed, 3 insertions, 5 deletions
diff --git a/theories/QArith/Qcanon.v b/theories/QArith/Qcanon.v
index 2ab27abaa..218289a4f 100644
--- a/theories/QArith/Qcanon.v
+++ b/theories/QArith/Qcanon.v
@@ -466,18 +466,16 @@ Proof.
destruct n; simpl.
destruct 1; auto.
intros.
- apply Qc_is_canon.
- simpl.
- compute; auto.
+ now apply Qc_is_canon.
Qed.
Lemma Qcpower_pos : forall p n, 0 <= p -> 0 <= p^n.
Proof.
induction n; simpl; auto with qarith.
- intros; compute; intro; discriminate.
+ easy.
intros.
apply Qcle_trans with (0*(p^n)).
- compute; intro; discriminate.
+ easy.
apply Qcmult_le_compat_r; auto.
Qed.