summaryrefslogtreecommitdiff
path: root/theories/Reals/Rtrigo_reg.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Reals/Rtrigo_reg.v')
-rw-r--r--theories/Reals/Rtrigo_reg.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Reals/Rtrigo_reg.v b/theories/Reals/Rtrigo_reg.v
index 9d3b60c6..1c9a9445 100644
--- a/theories/Reals/Rtrigo_reg.v
+++ b/theories/Reals/Rtrigo_reg.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id: Rtrigo_reg.v,v 1.15.2.1 2004/07/16 19:31:15 herbelin Exp $ i*)
+(*i $Id: Rtrigo_reg.v 8670 2006-03-28 22:16:14Z herbelin $ i*)
Require Import Rbase.
Require Import Rfunctions.
@@ -32,7 +32,7 @@ cut
(fun n:nat =>
sum_f_R0 (fun k:nat => Rabs (/ INR (fact (2 * k)) * r ^ (2 * k)))
n) l)).
-intro; elim X; intros.
+intro X; elim X; intros.
apply existT with x.
split.
apply p.
@@ -206,7 +206,7 @@ cut
sum_f_R0
(fun k:nat => Rabs (/ INR (fact (2 * k + 1)) * r ^ (2 * k))) n)
l)).
-intro; elim X; intros.
+intro X; elim X; intros.
apply existT with x.
split.
apply p.
@@ -605,4 +605,4 @@ Lemma derive_pt_cos :
forall x:R, derive_pt cos x (derivable_pt_cos _) = - sin x.
intros; apply derive_pt_eq_0.
apply derivable_pt_lim_cos.
-Qed. \ No newline at end of file
+Qed.