diff -r 5c8a0580d513 -r df976eefcba0 src/HOL/Complex_Analysis/Conformal_Mappings.thy --- a/src/HOL/Complex_Analysis/Conformal_Mappings.thy Thu Jul 15 22:51:49 2021 +0200 +++ b/src/HOL/Complex_Analysis/Conformal_Mappings.thy Fri Jul 16 14:43:25 2021 +0100 @@ -82,6 +82,38 @@ thus ?thesis by simp qed +corollary analytic_continuation': + assumes "f holomorphic_on S" "open S" "connected S" + and "U \ S" "\ \ S" "\ islimpt U" + and "f constant_on U" + shows "f constant_on S" +proof - + obtain c where c: "\x. x \ U \ f x - c = 0" + by (metis \f constant_on U\ constant_on_def diff_self) + have "(\z. f z - c) holomorphic_on S" + using assms by (intro holomorphic_intros) + with c analytic_continuation assms have "\x. x \ S \ f x - c = 0" + by blast + then show ?thesis + unfolding constant_on_def by force +qed + +lemma holomorphic_compact_finite_zeros: + assumes S: "f holomorphic_on S" "open S" "connected S" + and "compact K" "K \ S" + and "\ f constant_on S" + shows "finite {z\K. f z = 0}" +proof (rule ccontr) + assume "infinite {z\K. f z = 0}" + then obtain z where "z \ K" and z: "z islimpt {z\K. f z = 0}" + using \compact K\ by (auto simp: compact_eq_Bolzano_Weierstrass) + moreover have "{z\K. f z = 0} \ S" + using \K \ S\ by blast + ultimately show False + using assms analytic_continuation [OF S] unfolding constant_on_def + by blast +qed + subsection\Open mapping theorem\ lemma holomorphic_contract_to_zero: