diff options
author | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-06-29 10:10:14 +0000 |
---|---|---|
committer | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-06-29 10:10:14 +0000 |
commit | b66127f53f411da94048e8a98e745c642cb1c851 (patch) | |
tree | 5d1ac9502df9f27777259e178d860297b4f8c2db /plugins | |
parent | 4dce356eacb7b9804c2e2398447dbbc3b0dc1383 (diff) |
QArith: typo in name of hint db (fix #2346)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13220 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins')
-rw-r--r-- | plugins/micromega/QMicromega.v | 5 |
1 files changed, 0 insertions, 5 deletions
diff --git a/plugins/micromega/QMicromega.v b/plugins/micromega/QMicromega.v index ae22b0c78..1e909cbca 100644 --- a/plugins/micromega/QMicromega.v +++ b/plugins/micromega/QMicromega.v @@ -31,13 +31,8 @@ Proof. rewrite <- H ; rewrite <- H0 ; auto. rewrite H ; rewrite H0 ; auto. apply Qsrt. - apply Qle_refl. - apply Qle_antisym ; auto. eapply Qle_trans ; eauto. - apply Qlt_le_weak ; auto. apply (Qlt_not_eq n m H H0) ; auto. - destruct (Qle_lt_or_eq _ _ H0) ; auto. - tauto. destruct(Q_dec n m) as [[H1 |H1] | H1 ] ; tauto. apply (Qplus_le_compat p p n m (Qle_refl p) H). generalize (Qmult_lt_compat_r 0 n m H0 H). |