aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Alembert.v
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-03-06 17:51:49 +0100
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-03-06 17:51:49 +0100
commit21e439b65eab694adaccfaa39aec9415da0a4609 (patch)
tree59dc6958cac0c9e303467d3d1402a60cc8a90bfc /theories/Reals/Alembert.v
parent0b660db0a7d771ee8e165327cb954013bbc1a7c8 (diff)
Add some missing Proof keywords.
Diffstat (limited to 'theories/Reals/Alembert.v')
-rw-r--r--theories/Reals/Alembert.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/Reals/Alembert.v b/theories/Reals/Alembert.v
index e848e4df8..011328ec0 100644
--- a/theories/Reals/Alembert.v
+++ b/theories/Reals/Alembert.v
@@ -572,6 +572,7 @@ Lemma Alembert_C6 :
(forall n:nat, An n <> 0) ->
Un_cv (fun n:nat => Rabs (An (S n) / An n)) k ->
Rabs x < / k -> { l:R | Pser An x l }.
+Proof.
intros.
cut { l:R | Un_cv (fun N:nat => sum_f_R0 (fun i:nat => An i * x ^ i) N) l }.
intro X.