src/HOL/Probability/Sinc_Integral.thy
changeset 70532 fcf3b891ccb1
parent 70365 4df0628e8545
child 75462 7448423e5dba
--- a/src/HOL/Probability/Sinc_Integral.thy	Wed Aug 14 19:50:23 2019 +0200
+++ b/src/HOL/Probability/Sinc_Integral.thy	Thu Aug 15 16:11:56 2019 +0100
@@ -271,7 +271,7 @@
 
 lemma Si_at_top: "(Si \<longlongrightarrow> pi / 2) at_top"
 proof -
-  have "\<forall>\<^sub>F t in at_top. pi / 2 - (LBINT u=0..\<infinity>. exp (-(u * t)) * (u * sin t + cos t) / (1 + u^2)) = Si t"
+  have \<dagger>: "\<forall>\<^sub>F t in at_top. pi / 2 - (LBINT u=0..\<infinity>. exp (-(u * t)) * (u * sin t + cos t) / (1 + u^2)) = Si t"
     using eventually_ge_at_top[of 0]
   proof eventually_elim
     fix t :: real assume "t \<ge> 0"
@@ -326,8 +326,8 @@
       using Si_at_top_integrable[OF \<open>0\<le>t\<close>] by (simp add: integrable_I0i_1_div_plus_square LBINT_I0i_1_div_plus_square)
     finally show "pi / 2 - (LBINT u=0..\<infinity>. exp (-(u * t)) * (u * sin t + cos t) / (1 + u^2)) = Si t" ..
   qed
-  then show ?thesis
-    by (rule Lim_transform_eventually)
+  show ?thesis
+    by (rule Lim_transform_eventually [OF _ \<dagger>])
        (auto intro!: tendsto_eq_intros Si_at_top_LBINT)
 qed