src/HOL/Analysis/Summation_Tests.thy
changeset 68532 f8b98d31ad45
parent 66672 75694b28ef08
child 68643 3db6c9338ec1
--- a/src/HOL/Analysis/Summation_Tests.thy	Thu Jun 28 14:14:05 2018 +0100
+++ b/src/HOL/Analysis/Summation_Tests.thy	Thu Jun 28 17:14:40 2018 +0100
@@ -752,7 +752,7 @@
   assumes lim: "(\<lambda>n. ereal (norm (f n) / norm (f (Suc n)))) \<longlonglongrightarrow> c"
   shows   "conv_radius f = c"
 proof (rule conv_radius_eqI')
-  show "c \<ge> 0" by (intro Lim_bounded2_ereal[OF lim]) simp_all
+  show "c \<ge> 0" by (intro Lim_bounded2[OF lim]) simp_all
 next
   fix r assume r: "0 < r" "ereal r < c"
   let ?l = "liminf (\<lambda>n. ereal (norm (f n * of_real r ^ n) / norm (f (Suc n) * of_real r ^ Suc n)))"