aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rbase.v
diff options
context:
space:
mode:
authorGravatar mayero <mayero@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-06-19 01:56:20 +0000
committerGravatar mayero <mayero@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-06-19 01:56:20 +0000
commit513194c5c3b270171933bcb7784946a09e732d14 (patch)
tree6b571dc2217363b523f1fcce500b9a28fe99b7a7 /theories/Reals/Rbase.v
parentb9b7500136380e2465c13af1fba1019fad0c2ebf (diff)
Oubli Save + je sais plus
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1792 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rbase.v')
-rw-r--r--theories/Reals/Rbase.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/theories/Reals/Rbase.v b/theories/Reals/Rbase.v
index f2603ca67..a9c26fa72 100644
--- a/theories/Reals/Rbase.v
+++ b/theories/Reals/Rbase.v
@@ -964,7 +964,7 @@ Rewrite (Rmult_sym x); Rewrite <- Rmult_assoc; Rewrite (Rmult_sym y (Rinv y));
Apply imp_not_Req; Right.
Red; Apply Rlt_trans with r2 := x; Auto with real.
Save.
-Hints Resolve Rlt_Rinv_R1 :reals.
+Hints Resolve Rlt_Rinv_R1 :real.
(*********************************************************)
(*s Greater *)
@@ -1461,6 +1461,7 @@ Intros;Cut `m<=n`.
Intro H0;Elim (IZR_le m n H0);Intro;Auto.
Generalize (eq_IZR m n H1);Intro;ElimType False;Omega.
Omega.
+Save.
Lemma one_IZR_lt1 : (z:Z)``-1<(IZR z)<1``->`z=0`.
Intros z (H1,H2).