src/HOL/Complex_Analysis/Conformal_Mappings.thy
changeset 73932 fd21b4a93043
parent 72259 25cf074a4188
child 74007 df976eefcba0
--- a/src/HOL/Complex_Analysis/Conformal_Mappings.thy	Fri Jun 18 15:03:12 2021 +0200
+++ b/src/HOL/Complex_Analysis/Conformal_Mappings.thy	Thu Jul 08 08:42:36 2021 +0200
@@ -852,7 +852,7 @@
     show "\<exists>B. \<forall>x. B \<le> cmod x \<longrightarrow> dist ((inverse \<circ> f) x) 0 \<le> e"
       apply simp
       apply (clarsimp simp add: compact_eq_bounded_closed bounded_pos norm_inverse)
-      by (metis (no_types, hide_lams) inverse_inverse_eq le_less_trans less_eq_real_def less_imp_inverse_less linordered_field_no_ub not_less)
+      by (metis (no_types, opaque_lifting) inverse_inverse_eq le_less_trans less_eq_real_def less_imp_inverse_less linordered_field_no_ub not_less)
   qed
   then obtain a n where "\<And>z. f z = (\<Sum>i\<le>n. a i * z^i)"
     using assms pole_at_infinity by blast