diff -r 29032b496f2e -r c6b50597abbc src/HOL/Complex_Analysis/Complex_Singularities.thy --- a/src/HOL/Complex_Analysis/Complex_Singularities.thy Thu Feb 16 10:42:39 2023 +0000 +++ b/src/HOL/Complex_Analysis/Complex_Singularities.thy Thu Feb 16 12:21:21 2023 +0000 @@ -249,6 +249,12 @@ shows "not_essential f z \ not_essential g z'" unfolding not_essential_def using assms filterlim_cong is_pole_cong by fastforce +lemma not_essential_compose_iff: + assumes "filtermap g (at z) = at z'" + shows "not_essential (f \ g) z = not_essential f z'" + unfolding not_essential_def filterlim_def filtermap_compose assms is_pole_compose_iff[OF assms] + by blast + lemma isolated_singularity_at_cong: assumes "eventually (\x. f x = g x) (at z)" "z = z'" shows "isolated_singularity_at f z \ isolated_singularity_at g z'" @@ -362,8 +368,8 @@ ultimately have "(f' \ 0) F" unfolding F_def by (simp add: continuous_within) moreover have "(g \ g z) F" - using holomorphic_on_imp_continuous_on[OF g_holo,unfolded continuous_on_def] \r>0\ - unfolding F_def by auto + unfolding F_def + using \r>0\ centre_in_ball continuous_on_def g_holo holomorphic_on_imp_continuous_on by blast ultimately show " ((\w. f' w * g w) \ 0) F" using tendsto_mult by fastforce qed moreover have "(h \ h z) (at z within ball z r)" @@ -1058,7 +1064,7 @@ using analytic_at not_is_pole_holomorphic by blast lemma not_essential_const [singularity_intros]: "not_essential (\_. c) z" - unfolding not_essential_def by (rule exI[of _ c]) auto + by blast lemma not_essential_uminus [singularity_intros]: assumes f_ness: "not_essential f z"