src/HOL/Analysis/Conformal_Mappings.thy
changeset 63928 d81fb5b46a5c
parent 63918 6bf55e6e0b75
child 64267 b9a1486e79be
equal deleted inserted replaced
63927:0efb482beb84 63928:d81fb5b46a5c
  1025   qed
  1025   qed
  1026   have "bounded {z. (\<Sum>i\<le>n. c i * z ^ i) \<in> K}"
  1026   have "bounded {z. (\<Sum>i\<le>n. c i * z ^ i) \<in> K}"
  1027     using polyfun_extremal [where c=c and B="B+1", OF c]
  1027     using polyfun_extremal [where c=c and B="B+1", OF c]
  1028     by (auto simp: bounded_pos eventually_at_infinity_pos *)
  1028     by (auto simp: bounded_pos eventually_at_infinity_pos *)
  1029   moreover have "closed {z. (\<Sum>i\<le>n. c i * z ^ i) \<in> K}"
  1029   moreover have "closed {z. (\<Sum>i\<le>n. c i * z ^ i) \<in> K}"
  1030     apply (rule allI continuous_closed_preimage_univ continuous_intros)+
  1030     apply (intro allI continuous_closed_preimage_univ continuous_intros)
  1031     using \<open>compact K\<close> compact_eq_bounded_closed by blast
  1031     using \<open>compact K\<close> compact_eq_bounded_closed by blast
  1032   ultimately show ?thesis
  1032   ultimately show ?thesis
  1033     using closed_Int_compact [OF \<open>closed S\<close>] compact_eq_bounded_closed by blast
  1033     using closed_Int_compact [OF \<open>closed S\<close>] compact_eq_bounded_closed by blast
  1034 qed
  1034 qed
  1035 
  1035