aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rsqrt_def.v
diff options
context:
space:
mode:
authorGravatar desmettr <desmettr@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-01-22 16:46:36 +0000
committerGravatar desmettr <desmettr@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-01-22 16:46:36 +0000
commit9aeaac7698c670cc7ac92dd53cd674b5b321aab3 (patch)
treeb02945c21c26e6c67d0e17175bfb0e3f52b89f5c /theories/Reals/Rsqrt_def.v
parent096310efb4266fe89455d473f704ec6c7ed5a97c (diff)
Modifications dans SeqProp
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3590 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rsqrt_def.v')
-rw-r--r--theories/Reals/Rsqrt_def.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/theories/Reals/Rsqrt_def.v b/theories/Reals/Rsqrt_def.v
index ed939426f..8c63c9eb5 100644
--- a/theories/Reals/Rsqrt_def.v
+++ b/theories/Reals/Rsqrt_def.v
@@ -111,11 +111,11 @@ Assumption.
Apply le_O_n.
Qed.
-Lemma dicho_lb_maj : (x,y:R;P:R->bool) ``x<=y`` -> (majoree (dicho_lb x y P)).
+Lemma dicho_lb_maj : (x,y:R;P:R->bool) ``x<=y`` -> (has_ub (dicho_lb x y P)).
Intros.
Cut (n:nat)``(dicho_lb x y P n)<=y``.
Intro.
-Unfold majoree.
+Unfold has_ub.
Unfold bound.
Exists y.
Unfold is_upper_bound.
@@ -145,18 +145,18 @@ Assumption.
Assumption.
Qed.
-Lemma dicho_up_min : (x,y:R;P:R->bool) ``x<=y`` -> (minoree (dicho_up x y P)).
+Lemma dicho_up_min : (x,y:R;P:R->bool) ``x<=y`` -> (has_lb (dicho_up x y P)).
Intros.
Cut (n:nat)``x<=(dicho_up x y P n)``.
Intro.
-Unfold minoree.
+Unfold has_lb.
Unfold bound.
Exists ``-x``.
Unfold is_upper_bound.
Intros.
Elim H1; Intros.
Rewrite H2.
-Unfold opp_sui.
+Unfold opp_seq.
Apply Rle_Ropp1.
Apply H0.
Apply dicho_up_min_x; Assumption.
@@ -287,7 +287,7 @@ Intros.
Assert H2 := (CV_minus ? ? ? ? H0 H1).
Cut (Un_cv [i:nat]``(dicho_lb x y P i)-(dicho_up x y P i)`` R0).
Intro.
-Assert H4 := (UL_suite ? ? ? H2 H3).
+Assert H4 := (UL_sequence ? ? ? H2 H3).
Symmetry; Apply Rminus_eq_right; Assumption.
Unfold Un_cv; Unfold R_dist.
Intros.