src/HOL/Analysis/Infinite_Products.thy
changeset 70365 4df0628e8545
parent 70136 f03a01a18c6e
child 70817 dd675800469d
--- a/src/HOL/Analysis/Infinite_Products.thy	Thu Jul 11 18:37:52 2019 +0200
+++ b/src/HOL/Analysis/Infinite_Products.thy	Wed Jul 17 14:02:42 2019 +0100
@@ -1673,7 +1673,7 @@
     by (force simp add: eventually_sequentially intro: that)
   qed
   with \<theta>to\<Theta> have "(\<lambda>n. (\<Sum>j\<le>n. Im (Ln (z j)))) \<longlonglongrightarrow> \<Theta> + of_int K * (2*pi)"
-    by (simp add: k tendsto_add tendsto_mult Lim_eventually)
+    by (simp add: k tendsto_add tendsto_mult tendsto_eventually)
   moreover have "(\<lambda>n. (\<Sum>k\<le>n. Re (Ln (z k)))) \<longlonglongrightarrow> Re (Ln \<xi>)"
     using assms continuous_imp_tendsto [OF isCont_ln tendsto_norm [OF L]]
     by (simp add: o_def flip: prod_norm ln_prod)