summaryrefslogtreecommitdiff
path: root/theories/Reals/Exp_prop.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Reals/Exp_prop.v')
-rw-r--r--theories/Reals/Exp_prop.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Reals/Exp_prop.v b/theories/Reals/Exp_prop.v
index fcaeb11e..90ea93ef 100644
--- a/theories/Reals/Exp_prop.v
+++ b/theories/Reals/Exp_prop.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i $Id: Exp_prop.v,v 1.16.2.1 2004/07/16 19:31:10 herbelin Exp $ i*)
+(*i $Id: Exp_prop.v 8670 2006-03-28 22:16:14Z herbelin $ i*)
Require Import Rbase.
Require Import Rfunctions.
@@ -895,7 +895,7 @@ cut
Un_cv
(fun n:nat =>
sum_f_R0 (fun k:nat => Rabs (r ^ k / INR (fact (S k)))) n) l)).
-intro.
+intro X.
elim X; intros.
exists x; intros.
split.
@@ -1008,4 +1008,4 @@ rewrite Rmult_minus_distr_l.
rewrite Rmult_1_r; unfold Rdiv in |- *; rewrite <- Rmult_assoc;
rewrite Rmult_minus_distr_l.
rewrite Rmult_1_r; rewrite exp_plus; reflexivity.
-Qed. \ No newline at end of file
+Qed.