aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rseries.v
diff options
context:
space:
mode:
authorGravatar gmelquio <gmelquio@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-18 19:31:45 +0000
committerGravatar gmelquio <gmelquio@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-02-18 19:31:45 +0000
commit737d1b8008783e0c558065ca0836412f0c9b0e0d (patch)
tree4669a7057fbdeb7f487b9fd8fc2113bd43855092 /theories/Reals/Rseries.v
parentaef3d0dceedcc277b7b5128018b0beffd31601a8 (diff)
Removed SeqProp's dependency on Classical.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12796 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rseries.v')
-rw-r--r--theories/Reals/Rseries.v16
1 files changed, 11 insertions, 5 deletions
diff --git a/theories/Reals/Rseries.v b/theories/Reals/Rseries.v
index 15f02c69b..1ed6b03c5 100644
--- a/theories/Reals/Rseries.v
+++ b/theories/Reals/Rseries.v
@@ -100,12 +100,9 @@ Section sequence.
Qed.
(*********)
- Lemma Un_cv_crit : Un_growing -> bound EUn -> exists l : R, Un_cv l.
+ Lemma Un_cv_crit_lub : Un_growing -> forall l, is_lub EUn l -> Un_cv l.
Proof.
- intros Hug Heub.
- destruct (completeness EUn Heub EUn_noempty) as (l, H).
- exists l.
- intros eps Heps.
+ intros Hug l H eps Heps.
cut (exists N, Un N > l - eps).
intros (N, H3).
@@ -263,6 +260,15 @@ Section sequence.
Qed.
(*********)
+ Lemma Un_cv_crit : Un_growing -> bound EUn -> exists l : R, Un_cv l.
+ Proof.
+ intros Hug Heub.
+ exists (projT1 (completeness EUn Heub EUn_noempty)).
+ destruct (completeness EUn Heub EUn_noempty) as (l, H).
+ now apply Un_cv_crit_lub.
+ Qed.
+
+(*********)
Lemma finite_greater :
forall N:nat, exists M : R, (forall n:nat, (n <= N)%nat -> Un n <= M).
Proof.