src/HOL/Analysis/Complex_Analysis_Basics.thy
changeset 71001 3e374c65f96b
parent 70817 dd675800469d
child 71029 934e0044e94b
--- a/src/HOL/Analysis/Complex_Analysis_Basics.thy	Sat Nov 02 14:31:48 2019 +0000
+++ b/src/HOL/Analysis/Complex_Analysis_Basics.thy	Sat Nov 02 15:52:47 2019 +0000
@@ -5,7 +5,7 @@
 section \<open>Complex Analysis Basics\<close>
 
 theory Complex_Analysis_Basics
-  imports Brouwer_Fixpoint "HOL-Library.Nonpos_Ints"
+  imports Derivative "HOL-Library.Nonpos_Ints"
 begin
 
 (* TODO FIXME: A lot of the things in here have nothing to do with complex analysis *)
@@ -880,32 +880,6 @@
   apply (auto simp:  bounded_linear_mult_right)
   done
 
-lemma has_field_derivative_inverse_strong:
-  fixes f :: "'a::{euclidean_space,real_normed_field} \<Rightarrow> 'a"
-  shows "DERIV f x :> f' \<Longrightarrow>
-         f' \<noteq> 0 \<Longrightarrow>
-         open S \<Longrightarrow>
-         x \<in> S \<Longrightarrow>
-         continuous_on S f \<Longrightarrow>
-         (\<And>z. z \<in> S \<Longrightarrow> g (f z) = z)
-         \<Longrightarrow> DERIV g (f x) :> inverse (f')"
-  unfolding has_field_derivative_def
-  apply (rule has_derivative_inverse_strong [of S x f g ])
-  by auto
-
-lemma has_field_derivative_inverse_strong_x:
-  fixes f :: "'a::{euclidean_space,real_normed_field} \<Rightarrow> 'a"
-  shows  "DERIV f (g y) :> f' \<Longrightarrow>
-          f' \<noteq> 0 \<Longrightarrow>
-          open S \<Longrightarrow>
-          continuous_on S f \<Longrightarrow>
-          g y \<in> S \<Longrightarrow> f(g y) = y \<Longrightarrow>
-          (\<And>z. z \<in> S \<Longrightarrow> g (f z) = z)
-          \<Longrightarrow> DERIV g y :> inverse (f')"
-  unfolding has_field_derivative_def
-  apply (rule has_derivative_inverse_strong_x [of S g y f])
-  by auto
-
 subsection\<^marker>\<open>tag unimportant\<close> \<open>Taylor on Complex Numbers\<close>
 
 lemma sum_Suc_reindex: