aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rbase.v
diff options
context:
space:
mode:
authorGravatar desmettr <desmettr@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-01-15 15:35:04 +0000
committerGravatar desmettr <desmettr@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-01-15 15:35:04 +0000
commitfea0a3265a7191a7e8c13028e7edd9bf29ba4d25 (patch)
treef0993cfb172fd6e3cd280fcebf61ac0d6dc3e71b /theories/Reals/Rbase.v
parentd72eb6e333f710bb8f4ea0061e8399aafba19fe0 (diff)
Nouvelle interprétation des nombres réels
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3499 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rbase.v')
-rw-r--r--theories/Reals/Rbase.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Reals/Rbase.v b/theories/Reals/Rbase.v
index 11203d5ba..09dadee90 100644
--- a/theories/Reals/Rbase.v
+++ b/theories/Reals/Rbase.v
@@ -1508,7 +1508,7 @@ Qed.
Lemma double_var : (x:R) ``x == x/2 + x/2``.
Intro; Rewrite <- double; Unfold Rdiv; Rewrite <- Rmult_assoc; Symmetry; Apply Rinv_r_simpl_m.
-Replace ``2`` with (INR (2)); [Apply not_O_INR; Discriminate | Reflexivity].
+Replace ``2`` with (INR (2)); [Apply not_O_INR; Discriminate | Unfold INR; Ring].
Qed.
(**********************************************************)
@@ -1597,4 +1597,4 @@ Qed.
(**********)
Lemma complet_weak : (E:R->Prop) (bound E) -> (ExT [x:R] (E x)) -> (ExT [m:R] (is_lub E m)).
Intros; Elim (complet E H H0); Intros; Split with x; Assumption.
-Qed.
+Qed. \ No newline at end of file