src/HOL/Probability/Sinc_Integral.thy
changeset 62087 44841d07ef1d
parent 62083 7582b39f51ed
child 62390 842917225d56
--- a/src/HOL/Probability/Sinc_Integral.thy	Wed Jan 06 16:17:50 2016 +0100
+++ b/src/HOL/Probability/Sinc_Integral.thy	Thu Jan 07 17:40:55 2016 +0000
@@ -126,7 +126,7 @@
     by (auto simp: isCont_def sinc_at_0)
 next
   assume "x \<noteq> 0" show ?thesis
-    by (rule continuous_transform_at [where d = "abs x" and f = "\<lambda>x. sin x / x"])
+    by (rule continuous_transform_within [where d = "abs x" and f = "\<lambda>x. sin x / x"])
        (auto simp add: dist_real_def \<open>x \<noteq> 0\<close>)
 qed