src/HOL/Analysis/Conformal_Mappings.thy
changeset 63928 d81fb5b46a5c
parent 63918 6bf55e6e0b75
child 64267 b9a1486e79be
--- a/src/HOL/Analysis/Conformal_Mappings.thy	Wed Sep 21 14:20:07 2016 +0100
+++ b/src/HOL/Analysis/Conformal_Mappings.thy	Wed Sep 21 16:59:51 2016 +0100
@@ -1027,7 +1027,7 @@
     using polyfun_extremal [where c=c and B="B+1", OF c]
     by (auto simp: bounded_pos eventually_at_infinity_pos *)
   moreover have "closed {z. (\<Sum>i\<le>n. c i * z ^ i) \<in> K}"
-    apply (rule allI continuous_closed_preimage_univ continuous_intros)+
+    apply (intro allI continuous_closed_preimage_univ continuous_intros)
     using \<open>compact K\<close> compact_eq_bounded_closed by blast
   ultimately show ?thesis
     using closed_Int_compact [OF \<open>closed S\<close>] compact_eq_bounded_closed by blast