--- a/src/HOL/Complex_Analysis/Conformal_Mappings.thy Sat May 24 09:06:26 2025 +0200
+++ b/src/HOL/Complex_Analysis/Conformal_Mappings.thy Wed May 28 17:49:22 2025 +0200
@@ -723,7 +723,7 @@
then have "(\<lambda>z. if z = \<xi> then deriv g \<xi> else (g z - g \<xi>) / (z - \<xi>)) holomorphic_on S"
using \<xi> pole_lemma by blast
then show ?thesis
- using "\<section>" remove_def by fastforce
+ using "\<section>" by (smt (verit, best) DiffD2 singletonI)
qed
ultimately show "?P = ?Q" and "?P = ?R"
by meson+