src/HOL/Analysis/Cauchy_Integral_Theorem.thy
changeset 69712 dc85b5b3a532
parent 69661 a03a63b81f44
child 69922 4a9167f377b0
--- a/src/HOL/Analysis/Cauchy_Integral_Theorem.thy	Tue Jan 22 10:50:47 2019 +0000
+++ b/src/HOL/Analysis/Cauchy_Integral_Theorem.thy	Tue Jan 22 12:00:16 2019 +0000
@@ -3068,7 +3068,7 @@
     then have contfb: "continuous_on (ball z d) f"
       using contf continuous_on_subset by blast
     obtain h where "\<forall>y\<in>ball z d. (h has_field_derivative f y) (at y within ball z d)"
-      by (metis holomorphic_convex_primitive [OF convex_ball k contfb fcd] d interior_subset Diff_iff set_mp)
+      by (metis holomorphic_convex_primitive [OF convex_ball k contfb fcd] d interior_subset Diff_iff subsetD)
     then have "\<forall>y\<in>ball z d. (h has_field_derivative f y) (at y within s)"
       by (metis open_ball at_within_open d os subsetCE)
     then have "\<exists>h. (\<forall>y. cmod (y - z) < d \<longrightarrow> (h has_field_derivative f y) (at y within s))"