aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rlimit.v
diff options
context:
space:
mode:
authorGravatar mayero <mayero@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-05-07 15:33:42 +0000
committerGravatar mayero <mayero@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-05-07 15:33:42 +0000
commit578453f160673ab9dab97c30f564b7a9d9f16dae (patch)
tree4994af5a34127bc9714d5d983a91dc10d493ed3b /theories/Reals/Rlimit.v
parentd4815f9ccc6b59565f36cc5a4c66d9916728d202 (diff)
ex d'utilisation de fourier avec field
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1735 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Rlimit.v')
-rw-r--r--theories/Reals/Rlimit.v32
1 files changed, 2 insertions, 30 deletions
diff --git a/theories/Reals/Rlimit.v b/theories/Reals/Rlimit.v
index 471eb9f1c..3ebeccfdd 100644
--- a/theories/Reals/Rlimit.v
+++ b/theories/Reals/Rlimit.v
@@ -45,41 +45,13 @@ Save.
(*********)
Lemma Rlt_eps2_eps:(eps:R)(Rgt eps R0)->
(Rlt (Rmult eps (Rinv (Rplus R1 R1))) eps).
-Intros;Unfold Rgt in H;Pattern 2 eps;Rewrite <- Rmult_1r;
- Apply (Rlt_monotony eps (Rinv (Rplus R1 R1)) R1 H);
- Apply (Rlt_anti_compatibility (Rinv (Rplus R1 R1)) (Rinv (Rplus R1 R1))
- R1);Pattern 1 2 (Rinv (Rplus R1 R1));Rewrite <-Rmult_1l;
- Rewrite (eps2 R1);
- Pattern 1 R1;Rewrite <-Rplus_Or;
- Rewrite (Rplus_sym (Rinv (Rplus R1 R1)) R1);
- Apply (Rlt_compatibility R1 R0 (Rinv (Rplus R1 R1))
- (Rlt_Rinv (Rplus R1 R1) (Rlt_r_plus_R1 R1 (Rlt_le R0 R1 Rlt_R0_R1)))).
+Intros;Fourier.
Save.
(*********)
Lemma Rlt_eps4_eps:(eps:R)(Rgt eps R0)->
(Rlt (Rmult eps (Rinv (Rplus (Rplus R1 R1) (Rplus R1 R1)))) eps).
-Intros;Pattern 2 eps;Rewrite <-(let (H1,H2)=(Rmult_ne eps) in H1);
- Unfold Rgt in H;Apply Rlt_monotony;Auto.
- Generalize Rlt_R0_R1;Intro;
- Generalize (Rlt_compatibility R1 R0 R1 H0);Intro;
- Rewrite (let (H1,H2)=(Rplus_ne R1) in H1) in H1;
- Generalize (Rlt_compatibility R1 R1 (Rplus R1 R1) H1);Intro;
- Generalize (Rlt_compatibility (Rplus R1 R1) R1 (Rplus R1 R1) H1);Intro;
- Generalize (Rlt_trans R1 (Rplus R1 R1) (Rplus R1 (Rplus R1 R1))
- H1 H2);Intro;
- Rewrite (Rplus_sym (Rplus R1 R1) R1) in H3;
- Generalize (Rlt_trans R1 (Rplus R1 (Rplus R1 R1))
- (Rplus (Rplus R1 R1) (Rplus R1 R1)) H4 H3);Clear H H0 H1 H2 H3 H4;
- Intro;Rewrite <-(let (H1,H2)=(Rmult_ne
- (Rinv (Rplus (Rplus R1 R1) (Rplus R1 R1)))) in H1);Pattern 6 R1;
- Rewrite <-(Rinv_l (Rplus (Rplus R1 R1) (Rplus R1 R1))).
- Apply (Rlt_monotony (Rinv (Rplus (Rplus R1 R1) (Rplus R1 R1)))
- R1 (Rplus (Rplus R1 R1) (Rplus R1 R1)));Auto.
-Apply (Rlt_Rinv (Rplus (Rplus R1 R1) (Rplus R1 R1)));
- Apply (Rlt_trans R0 R1 (Rplus (Rplus R1 R1) (Rplus R1 R1)) Rlt_R0_R1 H).
-Apply (imp_not_Req (Rplus (Rplus R1 R1) (Rplus R1 R1)) R0);Right;Unfold Rgt;
- Apply (Rlt_trans R0 R1 (Rplus (Rplus R1 R1) (Rplus R1 R1)) Rlt_R0_R1 H).
+Intros;Fourier.
Save.
(*********)