src/HOL/Multivariate_Analysis/Cauchy_Integral_Thm.thy
changeset 62343 24106dc44def
parent 62217 527488dc8b90
child 62379 340738057c8c
--- a/src/HOL/Multivariate_Analysis/Cauchy_Integral_Thm.thy	Wed Feb 17 21:51:55 2016 +0100
+++ b/src/HOL/Multivariate_Analysis/Cauchy_Integral_Thm.thy	Wed Feb 17 21:51:56 2016 +0100
@@ -6690,7 +6690,7 @@
     using \<open>open s\<close>
     apply (simp add: open_contains_ball Ball_def)
     apply (erule all_forward)
-    using "*" by blast
+    using "*" by auto blast+
   have 2: "closedin (subtopology euclidean s) (\<Inter>n. {w \<in> s. (deriv ^^ n) f w = 0})"
     using assms
     by (auto intro: continuous_closed_in_preimage_constant holomorphic_on_imp_continuous_on holomorphic_higher_deriv)