src/HOL/Analysis/Conformal_Mappings.thy
changeset 70065 cc89a395b5a3
parent 69745 aec42cee2521
child 70113 c8deb8ba6d05
--- a/src/HOL/Analysis/Conformal_Mappings.thy	Fri Apr 05 11:22:00 2019 +0100
+++ b/src/HOL/Analysis/Conformal_Mappings.thy	Fri Apr 05 15:02:46 2019 +0100
@@ -3101,7 +3101,7 @@
       define f' where "f' \<equiv> \<lambda>x. (x - z) powr (n-m)"
       have "f' z=0" using \<open>n>m\<close> unfolding f'_def by auto
       moreover have "continuous F f'" unfolding f'_def F_def continuous_def
-        apply (subst netlimit_within)
+        apply (subst Lim_ident_at)
         using \<open>n>m\<close> by (auto intro!:tendsto_powr_complex_0 tendsto_eq_intros)  
       ultimately have "(f' \<longlongrightarrow> 0) F" unfolding F_def
         by (simp add: continuous_within)
@@ -3130,7 +3130,7 @@
       define f' where "f' \<equiv>\<lambda>x. (x - z) powr (m-n)"
       have "f' z=0" using \<open>m>n\<close> unfolding f'_def by auto
       moreover have "continuous F f'" unfolding f'_def F_def continuous_def
-        apply (subst netlimit_within)
+        apply (subst Lim_ident_at)
         using \<open>m>n\<close> by (auto intro!:tendsto_powr_complex_0 tendsto_eq_intros)
       ultimately have "(f' \<longlongrightarrow> 0) F" unfolding F_def
         by (simp add: continuous_within)