src/HOL/Complex_Analysis/Complex_Singularities.thy
author haftmann
Mon, 14 Apr 2025 20:19:05 +0200
changeset 82509 c476149a3790
parent 82310 41f5266e5595
child 82517 111b1b2a2d13
permissions -rw-r--r--
tuned
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     1
theory Complex_Singularities
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     2
  imports Conformal_Mappings
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     3
begin
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     4
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     5
subsection \<open>Non-essential singular points\<close>
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
     6
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
     7
definition\<^marker>\<open>tag important\<close>
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
     8
  is_pole :: "('a::topological_space \<Rightarrow> 'b::real_normed_vector) \<Rightarrow> 'a \<Rightarrow> bool" 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
     9
  where "is_pole f a =  (LIM x (at a). f x :> at_infinity)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    10
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    11
lemma is_pole_cong:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    12
  assumes "eventually (\<lambda>x. f x = g x) (at a)" "a=b"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    13
  shows "is_pole f a \<longleftrightarrow> is_pole g b"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    14
  unfolding is_pole_def using assms by (intro filterlim_cong,auto)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    15
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    16
lemma is_pole_transform:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    17
  assumes "is_pole f a" "eventually (\<lambda>x. f x = g x) (at a)" "a=b"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    18
  shows "is_pole g b"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    19
  using is_pole_cong assms by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    20
73795
8893e0ed263a new lemmas mostly about paths
paulson <lp15@cam.ac.uk>
parents: 72222
diff changeset
    21
lemma is_pole_shift_iff:
8893e0ed263a new lemmas mostly about paths
paulson <lp15@cam.ac.uk>
parents: 72222
diff changeset
    22
  fixes f :: "('a::real_normed_vector \<Rightarrow> 'b::real_normed_vector)"
8893e0ed263a new lemmas mostly about paths
paulson <lp15@cam.ac.uk>
parents: 72222
diff changeset
    23
  shows "is_pole (f \<circ> (+) d) a = is_pole f (a + d)"
8893e0ed263a new lemmas mostly about paths
paulson <lp15@cam.ac.uk>
parents: 72222
diff changeset
    24
  by (metis add_diff_cancel_right' filterlim_shift_iff is_pole_def)
8893e0ed263a new lemmas mostly about paths
paulson <lp15@cam.ac.uk>
parents: 72222
diff changeset
    25
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    26
lemma is_pole_tendsto:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
    27
  fixes f:: "('a::topological_space \<Rightarrow> 'b::real_normed_div_algebra)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    28
  shows "is_pole f x \<Longrightarrow> ((inverse o f) \<longlongrightarrow> 0) (at x)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    29
  unfolding is_pole_def
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
    30
  by (auto simp add: filterlim_inverse_at_iff[symmetric] comp_def filterlim_at)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    31
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    32
lemma is_pole_shift_0:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    33
  fixes f :: "('a::real_normed_vector \<Rightarrow> 'b::real_normed_vector)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    34
  shows "is_pole f z \<longleftrightarrow> is_pole (\<lambda>x. f (z + x)) 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    35
  unfolding is_pole_def by (subst at_to_0) (auto simp: filterlim_filtermap add_ac)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    36
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    37
lemma is_pole_shift_0':
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    38
  fixes f :: "('a::real_normed_vector \<Rightarrow> 'b::real_normed_vector)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    39
  shows "NO_MATCH 0 z \<Longrightarrow> is_pole f z \<longleftrightarrow> is_pole (\<lambda>x. f (z + x)) 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    40
  by (metis is_pole_shift_0)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    41
77228
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
    42
lemma is_pole_compose_iff:
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
    43
  assumes "filtermap g (at x) = (at y)"
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
    44
  shows   "is_pole (f \<circ> g) x \<longleftrightarrow> is_pole f y"
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
    45
  unfolding is_pole_def filterlim_def filtermap_compose assms ..
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
    46
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    47
lemma is_pole_inverse_holomorphic:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    48
  assumes "open s"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
    49
    and f_holo: "f holomorphic_on (s-{z})"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
    50
    and pole: "is_pole f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
    51
    and non_z: "\<forall>x\<in>s-{z}. f x\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    52
  shows "(\<lambda>x. if x=z then 0 else inverse (f x)) holomorphic_on s"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    53
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    54
  define g where "g \<equiv> \<lambda>x. if x=z then 0 else inverse (f x)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    55
  have "isCont g z" unfolding isCont_def  using is_pole_tendsto[OF pole]
72222
01397b6e5eb0 small quantifier fixes
paulson <lp15@cam.ac.uk>
parents: 71201
diff changeset
    56
    by (simp add: g_def cong: LIM_cong)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    57
  moreover have "continuous_on (s-{z}) f" using f_holo holomorphic_on_imp_continuous_on by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    58
  hence "continuous_on (s-{z}) (inverse o f)" unfolding comp_def
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
    59
    by (auto elim!:continuous_on_inverse simp add: non_z)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    60
  hence "continuous_on (s-{z}) g" unfolding g_def
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
    61
    using continuous_on_eq by fastforce
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    62
  ultimately have "continuous_on s g" using open_delete[OF \<open>open s\<close>] \<open>open s\<close>
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
    63
    by (auto simp add: continuous_on_eq_continuous_at)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    64
  moreover have "(inverse o f) holomorphic_on (s-{z})"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    65
    unfolding comp_def using f_holo
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
    66
    by (auto elim!:holomorphic_on_inverse simp add: non_z)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    67
  hence "g holomorphic_on (s-{z})"
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
    68
    using g_def holomorphic_transform by force
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    69
  ultimately show ?thesis unfolding g_def using \<open>open s\<close>
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    70
    by (auto elim!: no_isolated_singularity)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    71
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    72
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    73
lemma not_is_pole_holomorphic:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    74
  assumes "open A" "x \<in> A" "f holomorphic_on A"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    75
  shows   "\<not>is_pole f x"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    76
proof -
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    77
  have "continuous_on A f" 
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    78
    by (intro holomorphic_on_imp_continuous_on) fact
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    79
  with assms have "isCont f x" 
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    80
    by (simp add: continuous_on_eq_continuous_at)
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    81
  hence "f \<midarrow>x\<rightarrow> f x" 
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    82
    by (simp add: isCont_def)
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    83
  thus "\<not>is_pole f x" 
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    84
    unfolding is_pole_def
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    85
    using not_tendsto_and_filterlim_at_infinity[of "at x" f "f x"] by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    86
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    87
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    88
lemma is_pole_inverse_power: "n > 0 \<Longrightarrow> is_pole (\<lambda>z::complex. 1 / (z - a) ^ n) a"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    89
  unfolding is_pole_def inverse_eq_divide [symmetric]
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    90
  by (intro filterlim_compose[OF filterlim_inverse_at_infinity] tendsto_intros)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    91
     (auto simp: filterlim_at eventually_at intro!: exI[of _ 1] tendsto_eq_intros)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
    92
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    93
lemma is_pole_cmult_iff [simp]:
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    94
  assumes "c \<noteq> 0"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    95
  shows "is_pole (\<lambda>z. c * f z :: 'a :: real_normed_field) z \<longleftrightarrow> is_pole f z"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
    96
proof
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    97
  assume "is_pole (\<lambda>z. c * f z) z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    98
  with \<open>c\<noteq>0\<close> have "is_pole (\<lambda>z. inverse c * (c * f z)) z" 
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
    99
    unfolding is_pole_def
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   100
    by (force intro: tendsto_mult_filterlim_at_infinity)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   101
  thus "is_pole f z"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   102
    using \<open>c\<noteq>0\<close> by (simp add: field_simps)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   103
next
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   104
  assume "is_pole f z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   105
  with \<open>c\<noteq>0\<close> show "is_pole (\<lambda>z. c * f z) z"  
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   106
    by (auto intro!: tendsto_mult_filterlim_at_infinity simp: is_pole_def)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   107
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   108
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   109
lemma is_pole_uminus_iff [simp]: "is_pole (\<lambda>z. -f z :: 'a :: real_normed_field) z \<longleftrightarrow> is_pole f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   110
  using is_pole_cmult_iff[of "-1" f] by (simp del: is_pole_cmult_iff)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   111
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   112
lemma is_pole_inverse: "is_pole (\<lambda>z::complex. 1 / (z - a)) a"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   113
  using is_pole_inverse_power[of 1 a] by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   114
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   115
lemma is_pole_divide:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   116
  fixes f :: "'a :: t2_space \<Rightarrow> 'b :: real_normed_field"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   117
  assumes "isCont f z" "filterlim g (at 0) (at z)" "f z \<noteq> 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   118
  shows   "is_pole (\<lambda>z. f z / g z) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   119
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   120
  have "filterlim (\<lambda>z. f z * inverse (g z)) at_infinity (at z)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   121
    using assms filterlim_compose filterlim_inverse_at_infinity isCont_def
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   122
      tendsto_mult_filterlim_at_infinity by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   123
  thus ?thesis by (simp add: field_split_simps is_pole_def)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   124
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   125
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   126
lemma is_pole_basic:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   127
  assumes "f holomorphic_on A" "open A" "z \<in> A" "f z \<noteq> 0" "n > 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   128
  shows   "is_pole (\<lambda>w. f w / (w-z) ^ n) z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   129
proof (rule is_pole_divide)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   130
  have "continuous_on A f" by (rule holomorphic_on_imp_continuous_on) fact
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   131
  with assms show "isCont f z" by (auto simp: continuous_on_eq_continuous_at)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   132
  have "filterlim (\<lambda>w. (w-z) ^ n) (nhds 0) (at z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   133
    using assms by (auto intro!: tendsto_eq_intros)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   134
  thus "filterlim (\<lambda>w. (w-z) ^ n) (at 0) (at z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   135
    by (intro filterlim_atI tendsto_eq_intros)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   136
       (use assms in \<open>auto simp: eventually_at_filter\<close>)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   137
qed fact+
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   138
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   139
lemma is_pole_basic':
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   140
  assumes "f holomorphic_on A" "open A" "0 \<in> A" "f 0 \<noteq> 0" "n > 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   141
  shows   "is_pole (\<lambda>w. f w / w ^ n) 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   142
  using is_pole_basic[of f A 0] assms by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   143
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   144
lemma is_pole_compose: 
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   145
  assumes "is_pole f w" "g \<midarrow>z\<rightarrow> w" "eventually (\<lambda>z. g z \<noteq> w) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   146
  shows   "is_pole (\<lambda>x. f (g x)) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   147
  using assms(1) unfolding is_pole_def
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   148
  by (rule filterlim_compose) (use assms in \<open>auto simp: filterlim_at\<close>)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   149
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   150
lemma is_pole_plus_const_iff:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   151
  "is_pole f z \<longleftrightarrow> is_pole (\<lambda>x. f x + c) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   152
proof 
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   153
  assume "is_pole f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   154
  then have "filterlim f at_infinity (at z)" unfolding is_pole_def .
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   155
  moreover have "((\<lambda>_. c) \<longlongrightarrow> c) (at z)" by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   156
  ultimately have " LIM x (at z). f x + c :> at_infinity"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   157
    using tendsto_add_filterlim_at_infinity'[of f "at z"] by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   158
  then show "is_pole (\<lambda>x. f x + c) z" unfolding is_pole_def .
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   159
next
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   160
  assume "is_pole (\<lambda>x. f x + c) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   161
  then have "filterlim (\<lambda>x. f x + c) at_infinity (at z)" 
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   162
    unfolding is_pole_def .
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   163
  moreover have "((\<lambda>_. -c) \<longlongrightarrow> -c) (at z)" by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   164
  ultimately have "LIM x (at z). f x :> at_infinity"
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   165
    using tendsto_add_filterlim_at_infinity'[of "(\<lambda>x. f x + c)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   166
        "at z" "(\<lambda>_. - c)" "-c"] 
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   167
    by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   168
  then show "is_pole f z" unfolding is_pole_def .
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   169
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   170
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   171
lemma is_pole_minus_const_iff:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   172
  "is_pole (\<lambda>x. f x - c) z \<longleftrightarrow> is_pole f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   173
  using is_pole_plus_const_iff [of f z "-c"] by simp
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   174
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   175
lemma is_pole_alt:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   176
  "is_pole f x  = (\<forall>B>0. \<exists>U. open U \<and> x\<in>U \<and> (\<forall>y\<in>U. y\<noteq>x \<longrightarrow> norm (f y)\<ge>B))"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   177
  unfolding is_pole_def
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   178
  unfolding filterlim_at_infinity[of 0,simplified] eventually_at_topological
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   179
  by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   180
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   181
lemma is_pole_mult_analytic_nonzero1:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   182
  assumes "is_pole g x" "f analytic_on {x}" "f x \<noteq> 0"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   183
  shows   "is_pole (\<lambda>x. f x * g x) x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   184
  unfolding is_pole_def
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   185
proof (rule tendsto_mult_filterlim_at_infinity)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   186
  show "f \<midarrow>x\<rightarrow> f x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   187
    using assms by (simp add: analytic_at_imp_isCont isContD)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   188
qed (use assms in \<open>auto simp: is_pole_def\<close>)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   189
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   190
lemma is_pole_mult_analytic_nonzero2:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   191
  assumes "is_pole f x" "g analytic_on {x}" "g x \<noteq> 0"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   192
  shows   "is_pole (\<lambda>x. f x * g x) x"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   193
proof -
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   194
  have g: "g analytic_on {x}"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   195
    using assms by auto
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   196
  show ?thesis
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   197
    using is_pole_mult_analytic_nonzero1 [OF \<open>is_pole f x\<close> g] \<open>g x \<noteq> 0\<close>
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   198
    by (simp add: mult.commute)
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   199
qed
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   200
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   201
lemma is_pole_mult_analytic_nonzero1_iff:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   202
  assumes "f analytic_on {x}" "f x \<noteq> 0"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   203
  shows   "is_pole (\<lambda>x. f x * g x) x \<longleftrightarrow> is_pole g x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   204
proof
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   205
  assume "is_pole g x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   206
  thus "is_pole (\<lambda>x. f x * g x) x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   207
    by (intro is_pole_mult_analytic_nonzero1 assms)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   208
next
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   209
  assume "is_pole (\<lambda>x. f x * g x) x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   210
  hence "is_pole (\<lambda>x. inverse (f x) * (f x * g x)) x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   211
    by (rule is_pole_mult_analytic_nonzero1)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   212
       (use assms in \<open>auto intro!: analytic_intros\<close>)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   213
  also have "?this \<longleftrightarrow> is_pole g x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   214
  proof (rule is_pole_cong)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   215
    have "eventually (\<lambda>x. f x \<noteq> 0) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   216
      using assms by (simp add: analytic_at_neq_imp_eventually_neq)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   217
    thus "eventually (\<lambda>x. inverse (f x) * (f x * g x) = g x) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   218
      by eventually_elim auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   219
  qed auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   220
  finally show "is_pole g x" .
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   221
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   222
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   223
lemma is_pole_mult_analytic_nonzero2_iff:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   224
  assumes "g analytic_on {x}" "g x \<noteq> 0"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   225
  shows   "is_pole (\<lambda>x. f x * g x) x \<longleftrightarrow> is_pole f x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   226
  by (subst mult.commute, rule is_pole_mult_analytic_nonzero1_iff) (fact assms)+
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   227
77228
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   228
lemma frequently_const_imp_not_is_pole:
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   229
  fixes z :: "'a::first_countable_topology"
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   230
  assumes "frequently (\<lambda>w. f w = c) (at z)"
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   231
  shows   "\<not> is_pole f z"
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   232
proof
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   233
  assume "is_pole f z"
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   234
  from assms have "z islimpt {w. f w = c}"
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   235
    by (simp add: islimpt_conv_frequently_at)
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   236
  then obtain g where g: "\<And>n. g n \<in> {w. f w = c} - {z}" "g \<longlonglongrightarrow> z"
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   237
    unfolding islimpt_sequential by blast
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   238
  then have "(f \<circ> g) \<longlonglongrightarrow> c"
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   239
    by (simp add: tendsto_eventually)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   240
  moreover have "filterlim g (at z) sequentially"
77228
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   241
    using g by (auto simp: filterlim_at)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   242
  then have "filterlim (f \<circ> g) at_infinity sequentially"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   243
    unfolding o_def
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   244
    using \<open>is_pole f z\<close> filterlim_compose is_pole_def by blast
77228
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   245
  ultimately show False
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   246
    using not_tendsto_and_filterlim_at_infinity trivial_limit_sequentially by blast
8c093a4b8ccf Even more new material from Eberl and Li
paulson <lp15@cam.ac.uk>
parents: 77226
diff changeset
   247
qed
82310
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
   248
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
   249
subsection \<open>Isolated singularities\<close>
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
   250
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
   251
text \<open>The proposition
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   252
              \<^term>\<open>\<exists>x. ((f::complex\<Rightarrow>complex) \<longlongrightarrow> x) (at z) \<or> is_pole f z\<close>
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   253
can be interpreted as the complex function \<^term>\<open>f\<close> has a non-essential singularity at \<^term>\<open>z\<close>
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   254
(i.e. the singularity is either removable or a pole).\<close>
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   255
definition not_essential:: "[complex \<Rightarrow> complex, complex] \<Rightarrow> bool" where
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   256
  "not_essential f z = (\<exists>x. f\<midarrow>z\<rightarrow>x \<or> is_pole f z)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   257
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   258
definition isolated_singularity_at:: "[complex \<Rightarrow> complex, complex] \<Rightarrow> bool" where
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   259
  "isolated_singularity_at f z = (\<exists>r>0. f analytic_on ball z r-{z})"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   260
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   261
lemma not_essential_cong:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   262
  assumes "eventually (\<lambda>x. f x = g x) (at z)" "z = z'"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   263
  shows   "not_essential f z \<longleftrightarrow> not_essential g z'"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   264
  unfolding not_essential_def using assms filterlim_cong is_pole_cong by fastforce
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   265
77277
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 77228
diff changeset
   266
lemma not_essential_compose_iff:
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 77228
diff changeset
   267
  assumes "filtermap g (at z) = at z'"
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 77228
diff changeset
   268
  shows   "not_essential (f \<circ> g) z = not_essential f z'"
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 77228
diff changeset
   269
  unfolding not_essential_def filterlim_def filtermap_compose assms is_pole_compose_iff[OF assms]
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 77228
diff changeset
   270
  by blast
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 77228
diff changeset
   271
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   272
lemma isolated_singularity_at_cong:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   273
  assumes "eventually (\<lambda>x. f x = g x) (at z)" "z = z'"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   274
  shows   "isolated_singularity_at f z \<longleftrightarrow> isolated_singularity_at g z'"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   275
proof -
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   276
  have "isolated_singularity_at g z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   277
    if "isolated_singularity_at f z" "eventually (\<lambda>x. f x = g x) (at z)" for f g
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   278
  proof -
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   279
    from that(1) obtain r where r: "r > 0" "f analytic_on ball z r - {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   280
      by (auto simp: isolated_singularity_at_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   281
    from that(2) obtain r' where r': "r' > 0" "\<forall>x\<in>ball z r'-{z}. f x = g x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   282
      unfolding eventually_at_filter eventually_nhds_metric by (auto simp: dist_commute)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   283
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   284
    have "f holomorphic_on ball z r - {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   285
      using r(2) by (subst (asm) analytic_on_open) auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   286
    hence "f holomorphic_on ball z (min r r') - {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   287
      by (rule holomorphic_on_subset) auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   288
    also have "?this \<longleftrightarrow> g holomorphic_on ball z (min r r') - {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   289
      using r' by (intro holomorphic_cong) auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   290
    also have "\<dots> \<longleftrightarrow> g analytic_on ball z (min r r') - {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   291
      by (subst analytic_on_open) auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   292
    finally show ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   293
      unfolding isolated_singularity_at_def
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   294
      by (intro exI[of _ "min r r'"]) (use \<open>r > 0\<close> \<open>r' > 0\<close> in auto)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   295
  qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   296
  from this[of f g] this[of g f] assms show ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   297
    by (auto simp: eq_commute)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   298
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   299
  
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   300
lemma removable_singularity:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   301
  assumes "f holomorphic_on A - {x}" "open A"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   302
  assumes "f \<midarrow>x\<rightarrow> c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   303
  shows   "(\<lambda>y. if y = x then c else f y) holomorphic_on A" (is "?g holomorphic_on _")
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   304
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   305
  have "continuous_on A ?g"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   306
    unfolding continuous_on_def
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   307
  proof
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   308
    fix y assume y: "y \<in> A"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   309
    show "(?g \<longlongrightarrow> ?g y) (at y within A)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   310
    proof (cases "y = x")
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   311
      case False
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   312
      have "continuous_on (A - {x}) f"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   313
        using assms(1) by (meson holomorphic_on_imp_continuous_on)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   314
      hence "(f \<longlongrightarrow> ?g y) (at y within A - {x})"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   315
        using False y by (auto simp: continuous_on_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   316
      also have "?this \<longleftrightarrow> (?g \<longlongrightarrow> ?g y) (at y within A - {x})"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   317
        by (intro filterlim_cong refl) (auto simp: eventually_at_filter)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   318
      also have "at y within A - {x} = at y within A"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   319
        using y assms False
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   320
        by (intro at_within_nhd[of _ "A - {x}"]) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   321
      finally show ?thesis .
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   322
    next
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   323
      case [simp]: True
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   324
      have "f \<midarrow>x\<rightarrow> c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   325
        by fact
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   326
      also have "?this \<longleftrightarrow> (?g \<longlongrightarrow> ?g y) (at y)"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   327
        by (simp add: LIM_equal)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   328
      finally show ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   329
        by (meson Lim_at_imp_Lim_at_within)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   330
    qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   331
  qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   332
  moreover {
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   333
    have "?g holomorphic_on A - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   334
      using assms(1) holomorphic_transform by fastforce
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   335
  }
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   336
  ultimately show ?thesis
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   337
    using assms by (simp add: no_isolated_singularity)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   338
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   339
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   340
lemma removable_singularity':
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   341
  assumes "isolated_singularity_at f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   342
  assumes "f \<midarrow>z\<rightarrow> c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   343
  shows   "(\<lambda>y. if y = z then c else f y) analytic_on {z}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   344
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   345
  from assms obtain r where r: "r > 0" "f analytic_on ball z r - {z}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   346
    by (auto simp: isolated_singularity_at_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   347
  have "(\<lambda>y. if y = z then c else f y) holomorphic_on ball z r"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   348
  proof (rule removable_singularity)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   349
    show "f holomorphic_on ball z r - {z}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   350
      using r(2) by (subst (asm) analytic_on_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   351
  qed (use assms in auto)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   352
  thus ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   353
    using r(1) unfolding analytic_at by (intro exI[of _ "ball z r"]) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   354
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   355
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   356
named_theorems singularity_intros "introduction rules for singularities"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   357
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   358
lemma holomorphic_factor_unique:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   359
  fixes f:: "complex \<Rightarrow> complex" and z::complex and r::real and m n::int
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   360
  assumes "r>0" "g z\<noteq>0" "h z\<noteq>0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   361
    and asm: "\<forall>w\<in>ball z r-{z}. f w = g w * (w-z) powi n \<and> g w\<noteq>0 \<and> f w =  h w * (w-z) powi m \<and> h w\<noteq>0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   362
    and g_holo: "g holomorphic_on ball z r" and h_holo: "h holomorphic_on ball z r"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   363
  shows "n=m"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   364
proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   365
  have [simp]: "at z within ball z r \<noteq> bot" using \<open>r>0\<close>
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   366
      by (auto simp add: at_within_ball_bot_iff)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   367
  have False when "n>m"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   368
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   369
    have "(h \<longlongrightarrow> 0) (at z within ball z r)"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   370
    proof (rule Lim_transform_within[OF _ \<open>r>0\<close>, where f="\<lambda>w. (w-z) powi (n - m) * g w"])
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   371
      have "\<forall>w\<in>ball z r-{z}. h w = (w-z)powi(n-m) * g w"
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   372
        using \<open>n>m\<close> asm \<open>r>0\<close> by (simp add: field_simps power_int_diff) force
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   373
      then show "\<lbrakk>x' \<in> ball z r; 0 < dist x' z;dist x' z < r\<rbrakk>
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   374
            \<Longrightarrow> (x' - z) powi (n - m) * g x' = h x'" for x' by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   375
    next
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   376
      define F where "F \<equiv> at z within ball z r"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   377
      define f' where "f' \<equiv> \<lambda>x. (x - z) powi (n-m)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   378
      have "f' z=0" using \<open>n>m\<close> unfolding f'_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   379
      moreover have "continuous F f'" unfolding f'_def F_def continuous_def
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   380
        using \<open>n>m\<close>
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   381
          by (auto simp add: Lim_ident_at  intro!:tendsto_powr_complex_0 tendsto_eq_intros)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   382
      ultimately have "(f' \<longlongrightarrow> 0) F" unfolding F_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   383
        by (simp add: continuous_within)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   384
      moreover have "(g \<longlongrightarrow> g z) F"
77277
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 77228
diff changeset
   385
        unfolding F_def
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 77228
diff changeset
   386
        using \<open>r>0\<close> centre_in_ball continuous_on_def g_holo holomorphic_on_imp_continuous_on by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   387
      ultimately show " ((\<lambda>w. f' w * g w) \<longlongrightarrow> 0) F" using tendsto_mult by fastforce
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   388
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   389
    moreover have "(h \<longlongrightarrow> h z) (at z within ball z r)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   390
      using holomorphic_on_imp_continuous_on[OF h_holo]
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   391
      by (auto simp add: continuous_on_def \<open>r>0\<close>)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   392
    ultimately have "h z=0" by (auto intro!: tendsto_unique)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   393
    thus False using \<open>h z\<noteq>0\<close> by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   394
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   395
  moreover have False when "m>n"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   396
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   397
    have "(g \<longlongrightarrow> 0) (at z within ball z r)"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   398
    proof (rule Lim_transform_within[OF _ \<open>r>0\<close>, where f="\<lambda>w. (w-z) powi (m - n) * h w"])
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   399
      have "\<forall>w\<in>ball z r -{z}. g w = (w-z) powi (m-n) * h w" using \<open>m>n\<close> asm
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   400
        by (simp add: field_simps power_int_diff) force
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   401
      then show "\<lbrakk>x' \<in> ball z r; 0 < dist x' z;dist x' z < r\<rbrakk>
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   402
            \<Longrightarrow> (x' - z) powi (m - n) * h x' = g x'" for x' by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   403
    next
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   404
      define F where "F \<equiv> at z within ball z r"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   405
      define f' where "f' \<equiv>\<lambda>x. (x - z) powi (m-n)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   406
      have "f' z=0" using \<open>m>n\<close> unfolding f'_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   407
      moreover have "continuous F f'" unfolding f'_def F_def continuous_def
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   408
        using \<open>m>n\<close>
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   409
        by (auto simp: Lim_ident_at intro!:tendsto_powr_complex_0 tendsto_eq_intros)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   410
      ultimately have "(f' \<longlongrightarrow> 0) F" unfolding F_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   411
        by (simp add: continuous_within)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   412
      moreover have "(h \<longlongrightarrow> h z) F"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   413
        using holomorphic_on_imp_continuous_on[OF h_holo,unfolded continuous_on_def] \<open>r>0\<close>
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   414
        unfolding F_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   415
      ultimately show " ((\<lambda>w. f' w * h w) \<longlongrightarrow> 0) F" using tendsto_mult by fastforce
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   416
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   417
    moreover have "(g \<longlongrightarrow> g z) (at z within ball z r)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   418
      using holomorphic_on_imp_continuous_on[OF g_holo]
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   419
      by (auto simp add: continuous_on_def \<open>r>0\<close>)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   420
    ultimately have "g z=0" by (auto intro!: tendsto_unique)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   421
    thus False using \<open>g z\<noteq>0\<close> by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   422
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   423
  ultimately show "n=m" by fastforce
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   424
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   425
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   426
lemma holomorphic_factor_puncture:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   427
  assumes f_iso: "isolated_singularity_at f z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   428
      and "not_essential f z" \<comment> \<open>\<^term>\<open>f\<close> has either a removable singularity or a pole at \<^term>\<open>z\<close>\<close>
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   429
      and non_zero: "\<exists>\<^sub>Fw in (at z). f w\<noteq>0" \<comment> \<open>\<^term>\<open>f\<close> will not be constantly zero in a neighbour of \<^term>\<open>z\<close>\<close>
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   430
  shows "\<exists>!n::int. \<exists>g r. 0 < r \<and> g holomorphic_on cball z r \<and> g z\<noteq>0
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   431
          \<and> (\<forall>w\<in>cball z r-{z}. f w = g w * (w-z) powi n \<and> g w\<noteq>0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   432
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   433
  define P where "P = (\<lambda>f n g r. 0 < r \<and> g holomorphic_on cball z r \<and> g z\<noteq>0
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   434
          \<and> (\<forall>w\<in>cball z r - {z}. f w = g w * (w-z) powi n  \<and> g w\<noteq>0))"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   435
  have imp_unique: "\<exists>!n::int. \<exists>g r. P f n g r" when "\<exists>n g r. P f n g r"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   436
  proof (rule ex_ex1I[OF that])
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   437
    fix n1 n2 :: int
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   438
    assume g1_asm: "\<exists>g1 r1. P f n1 g1 r1" and g2_asm: "\<exists>g2 r2. P f n2 g2 r2"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   439
    define fac where "fac \<equiv> \<lambda>n g r. \<forall>w\<in>cball z r-{z}. f w = g w * (w-z) powi n \<and> g w \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   440
    obtain g1 r1 where "0 < r1" and g1_holo: "g1 holomorphic_on cball z r1" and "g1 z\<noteq>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   441
        and "fac n1 g1 r1" using g1_asm unfolding P_def fac_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   442
    obtain g2 r2 where "0 < r2" and g2_holo: "g2 holomorphic_on cball z r2" and "g2 z\<noteq>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   443
        and "fac n2 g2 r2" using g2_asm unfolding P_def fac_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   444
    define r where "r \<equiv> min r1 r2"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   445
    have "r>0" using \<open>r1>0\<close> \<open>r2>0\<close> unfolding r_def by auto
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   446
    moreover have "\<forall>w\<in>ball z r-{z}. f w = g1 w * (w-z) powi n1 \<and> g1 w\<noteq>0
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   447
        \<and> f w = g2 w * (w-z) powi n2  \<and> g2 w\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   448
      using \<open>fac n1 g1 r1\<close> \<open>fac n2 g2 r2\<close>   unfolding fac_def r_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   449
      by fastforce
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   450
    ultimately show "n1=n2" 
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   451
      using g1_holo g2_holo \<open>g1 z\<noteq>0\<close> \<open>g2 z\<noteq>0\<close>
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   452
      apply (elim holomorphic_factor_unique)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   453
      by (auto simp add: r_def)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   454
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   455
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   456
  have P_exist: "\<exists> n g r. P h n g r" when
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   457
      "\<exists>z'. (h \<longlongrightarrow> z') (at z)" "isolated_singularity_at h z"  "\<exists>\<^sub>Fw in (at z). h w\<noteq>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   458
    for h
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   459
  proof -
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   460
    from that(2) obtain r where "r>0" and r: "h analytic_on ball z r - {z}"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   461
      unfolding isolated_singularity_at_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   462
    obtain z' where "(h \<longlongrightarrow> z') (at z)" using \<open>\<exists>z'. (h \<longlongrightarrow> z') (at z)\<close> by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   463
    define h' where "h'=(\<lambda>x. if x=z then z' else h x)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   464
    have "h' holomorphic_on ball z r"
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   465
    proof (rule no_isolated_singularity'[of "{z}"])
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   466
      show "\<And>w. w \<in> {z} \<Longrightarrow> (h' \<longlongrightarrow> h' w) (at w within ball z r)"
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   467
        by (simp add: LIM_cong Lim_at_imp_Lim_at_within \<open>h \<midarrow>z\<rightarrow> z'\<close> h'_def)
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   468
      show "h' holomorphic_on ball z r - {z}"
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   469
        using r analytic_imp_holomorphic h'_def holomorphic_transform by fastforce
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   470
    qed auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   471
    have ?thesis when "z'=0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   472
    proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   473
      have "h' z=0" using that unfolding h'_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   474
      moreover have "\<not> h' constant_on ball z r"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   475
        using \<open>\<exists>\<^sub>Fw in (at z). h w\<noteq>0\<close> unfolding constant_on_def frequently_def eventually_at h'_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   476
        by (metis \<open>0 < r\<close> centre_in_ball dist_commute mem_ball that)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   477
      moreover note \<open>h' holomorphic_on ball z r\<close>
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   478
      ultimately obtain g r1 n where "0 < n" "0 < r1" "ball z r1 \<subseteq> ball z r" and
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   479
          g: "g holomorphic_on ball z r1"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   480
          "\<And>w. w \<in> ball z r1 \<Longrightarrow> h' w = (w-z) ^ n * g w"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   481
          "\<And>w. w \<in> ball z r1 \<Longrightarrow> g w \<noteq> 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   482
        using holomorphic_factor_zero_nonconstant[of _ "ball z r" z thesis,simplified,
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   483
                OF \<open>h' holomorphic_on ball z r\<close> \<open>r>0\<close> \<open>h' z=0\<close> \<open>\<not> h' constant_on ball z r\<close>]
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   484
        by (auto simp add: dist_commute)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   485
      define rr where "rr=r1/2"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   486
      have "P h' n g rr"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   487
        unfolding P_def rr_def
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   488
        using \<open>n>0\<close> \<open>r1>0\<close> g by (auto simp add: powr_nat)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   489
      then have "P h n g rr"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   490
        unfolding h'_def P_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   491
      then show ?thesis unfolding P_def by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   492
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   493
    moreover have ?thesis when "z'\<noteq>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   494
    proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   495
      have "h' z\<noteq>0" using that unfolding h'_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   496
      obtain r1 where "r1>0" "cball z r1 \<subseteq> ball z r" "\<forall>x\<in>cball z r1. h' x\<noteq>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   497
      proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   498
        have "isCont h' z" "h' z\<noteq>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   499
          by (auto simp add: Lim_cong_within \<open>h \<midarrow>z\<rightarrow> z'\<close> \<open>z'\<noteq>0\<close> continuous_at h'_def)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   500
        then obtain r2 where r2: "r2>0" "\<forall>x\<in>ball z r2. h' x\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   501
          using continuous_at_avoid[of z h' 0 ] unfolding ball_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   502
        define r1 where "r1=min r2 r / 2"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   503
        have "0 < r1" "cball z r1 \<subseteq> ball z r"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   504
          using \<open>r2>0\<close> \<open>r>0\<close> unfolding r1_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   505
        moreover have "\<forall>x\<in>cball z r1. h' x \<noteq> 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   506
          using r2 unfolding r1_def by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   507
        ultimately show ?thesis using that by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   508
      qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   509
      then have "P h' 0 h' r1" using \<open>h' holomorphic_on ball z r\<close> unfolding P_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   510
      then have "P h 0 h' r1" unfolding P_def h'_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   511
      then show ?thesis unfolding P_def by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   512
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   513
    ultimately show ?thesis by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   514
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   515
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   516
  have ?thesis when "\<exists>x. (f \<longlongrightarrow> x) (at z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   517
    apply (rule_tac imp_unique[unfolded P_def])
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   518
    using P_exist[OF that(1) f_iso non_zero] unfolding P_def .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   519
  moreover have ?thesis when "is_pole f z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   520
  proof (rule imp_unique[unfolded P_def])
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   521
    obtain e where [simp]: "e>0" and e_holo: "f holomorphic_on ball z e - {z}" and e_nz: "\<forall>x\<in>ball z e-{z}. f x\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   522
    proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   523
      have "\<forall>\<^sub>F z in at z. f z \<noteq> 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   524
        using \<open>is_pole f z\<close> filterlim_at_infinity_imp_eventually_ne unfolding is_pole_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   525
        by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   526
      then obtain e1 where e1: "e1>0" "\<forall>x\<in>ball z e1-{z}. f x\<noteq>0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   527
        using that eventually_at[of "\<lambda>x. f x\<noteq>0" z UNIV,simplified] by (auto simp add: dist_commute)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   528
      obtain e2 where e2: "e2>0" "f holomorphic_on ball z e2 - {z}"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   529
        using f_iso analytic_imp_holomorphic unfolding isolated_singularity_at_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   530
      show ?thesis
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   531
        using e1 e2 by (force intro: that[of "min e1 e2"])
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   532
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   533
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   534
    define h where "h \<equiv> \<lambda>x. inverse (f x)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   535
    have "\<exists>n g r. P h n g r"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   536
    proof -
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   537
      have "(\<lambda>x. inverse (f x)) analytic_on ball z e - {z}"
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   538
        by (metis e_holo e_nz open_ball analytic_on_open holomorphic_on_inverse open_delete)
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   539
      moreover have "h \<midarrow>z\<rightarrow> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   540
        using Lim_transform_within_open assms(2) h_def is_pole_tendsto that by fastforce
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   541
      moreover have "\<exists>\<^sub>Fw in (at z). h w\<noteq>0"
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   542
        using non_zero by (simp add: h_def)
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   543
      ultimately show ?thesis
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   544
        using P_exist[of h] \<open>e > 0\<close>
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   545
        unfolding isolated_singularity_at_def h_def
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   546
        by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   547
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   548
    then obtain n g r
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   549
      where "0 < r" and
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   550
            g_holo: "g holomorphic_on cball z r" and "g z\<noteq>0" and
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   551
            g_fac: "(\<forall>w\<in>cball z r-{z}. h w = g w * (w-z) powi n  \<and> g w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   552
      unfolding P_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   553
    have "P f (-n) (inverse o g) r"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   554
    proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   555
      have "f w = inverse (g w) * (w-z) powi (- n)" when "w\<in>cball z r - {z}" for w
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   556
        by (metis g_fac h_def inverse_inverse_eq inverse_mult_distrib power_int_minus that)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   557
      then show ?thesis
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   558
        unfolding P_def comp_def
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   559
        using \<open>r>0\<close> g_holo g_fac \<open>g z\<noteq>0\<close> by (auto intro: holomorphic_intros)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   560
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   561
    then show "\<exists>x g r. 0 < r \<and> g holomorphic_on cball z r \<and> g z \<noteq> 0
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   562
                  \<and> (\<forall>w\<in>cball z r - {z}. f w = g w * (w-z) powi x  \<and> g w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   563
      unfolding P_def by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   564
  qed
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   565
  ultimately show ?thesis 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   566
    using \<open>not_essential f z\<close> unfolding not_essential_def by presburger
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   567
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   568
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   569
lemma not_essential_transform:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   570
  assumes "not_essential g z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   571
  assumes "\<forall>\<^sub>F w in (at z). g w = f w"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   572
  shows "not_essential f z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   573
  using assms unfolding not_essential_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   574
  by (simp add: filterlim_cong is_pole_cong)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   575
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   576
lemma isolated_singularity_at_transform:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   577
  assumes "isolated_singularity_at g z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   578
  assumes "\<forall>\<^sub>F w in (at z). g w = f w"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   579
  shows "isolated_singularity_at f z"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   580
  using assms isolated_singularity_at_cong by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   581
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   582
lemma not_essential_powr[singularity_intros]:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   583
  assumes "LIM w (at z). f w :> (at x)"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   584
  shows "not_essential (\<lambda>w. (f w) powi n) z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   585
proof -
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   586
  define fp where "fp=(\<lambda>w. (f w) powi n)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   587
  have ?thesis when "n>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   588
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   589
    have "(\<lambda>w.  (f w) ^ (nat n)) \<midarrow>z\<rightarrow> x ^ nat n"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   590
      using that assms unfolding filterlim_at by (auto intro!:tendsto_eq_intros)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   591
    then have "fp \<midarrow>z\<rightarrow> x ^ nat n" unfolding fp_def
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   592
      by (smt (verit) LIM_cong power_int_def that)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   593
    then show ?thesis unfolding not_essential_def fp_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   594
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   595
  moreover have ?thesis when "n=0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   596
  proof -
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   597
    have "\<forall>\<^sub>F x in at z. fp x = 1"
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   598
      using that filterlim_at_within_not_equal[OF assms] by (auto simp: fp_def)
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   599
    then have "fp \<midarrow>z\<rightarrow> 1"
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   600
      by (simp add: tendsto_eventually)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   601
    then show ?thesis unfolding fp_def not_essential_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   602
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   603
  moreover have ?thesis when "n<0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   604
  proof (cases "x=0")
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   605
    case True
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   606
    have "(\<lambda>x. f x ^ nat (- n)) \<midarrow>z\<rightarrow> 0"
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   607
      using assms True that unfolding filterlim_at by (auto intro!:tendsto_eq_intros)
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   608
    moreover have "\<forall>\<^sub>F x in at z. f x ^ nat (- n) \<noteq> 0"
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   609
      by (smt (verit) True assms eventually_at_topological filterlim_at power_eq_0_iff)
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   610
    ultimately have "LIM w (at z). inverse ((f w) ^ (nat (-n))) :> at_infinity"
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   611
      by (metis filterlim_atI filterlim_compose filterlim_inverse_at_infinity)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   612
    then have "LIM w (at z). fp w :> at_infinity"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   613
    proof (elim filterlim_mono_eventually)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   614
      show "\<forall>\<^sub>F x in at z. inverse (f x ^ nat (- n)) = fp x"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   615
        using filterlim_at_within_not_equal[OF assms,of 0] unfolding fp_def
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   616
        by (smt (verit) eventuallyI power_int_def power_inverse that)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   617
    qed auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   618
    then show ?thesis unfolding fp_def not_essential_def is_pole_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   619
  next
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   620
    case False
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   621
    let ?xx= "inverse (x ^ (nat (-n)))"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   622
    have "(\<lambda>w. inverse ((f w) ^ (nat (-n)))) \<midarrow>z\<rightarrow>?xx"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   623
      using assms False unfolding filterlim_at by (auto intro!:tendsto_eq_intros)
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   624
    then have "fp \<midarrow>z\<rightarrow> ?xx"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   625
      by (smt (verit, best) LIM_cong fp_def power_int_def power_inverse that)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   626
    then show ?thesis unfolding fp_def not_essential_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   627
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   628
  ultimately show ?thesis by linarith
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   629
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   630
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   631
lemma isolated_singularity_at_powr[singularity_intros]:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   632
  assumes "isolated_singularity_at f z" "\<forall>\<^sub>F w in (at z). f w\<noteq>0"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   633
  shows "isolated_singularity_at (\<lambda>w. (f w) powi n) z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   634
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   635
  obtain r1 where "r1>0" "f analytic_on ball z r1 - {z}"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   636
    using assms(1) unfolding isolated_singularity_at_def by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   637
  then have r1: "f holomorphic_on ball z r1 - {z}"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   638
    using analytic_on_open[of "ball z r1-{z}" f] by blast
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   639
  obtain r2 where "r2>0" and r2: "\<forall>w. w \<noteq> z \<and> dist w z < r2 \<longrightarrow> f w \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   640
    using assms(2) unfolding eventually_at by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   641
  define r3 where "r3=min r1 r2"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   642
  have "(\<lambda>w. (f w) powi n) holomorphic_on ball z r3 - {z}"
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   643
    by (intro holomorphic_on_power_int) (use r1 r2 in \<open>auto simp: dist_commute r3_def\<close>)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   644
  moreover have "r3>0" unfolding r3_def using \<open>0 < r1\<close> \<open>0 < r2\<close> by linarith
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   645
  ultimately show ?thesis
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   646
    by (meson open_ball analytic_on_open isolated_singularity_at_def open_delete)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   647
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   648
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   649
lemma non_zero_neighbour:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   650
  assumes f_iso: "isolated_singularity_at f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   651
      and f_ness: "not_essential f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   652
      and f_nconst: "\<exists>\<^sub>Fw in (at z). f w\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   653
    shows "\<forall>\<^sub>F w in (at z). f w\<noteq>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   654
proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   655
  obtain fn fp fr
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   656
    where [simp]: "fp z \<noteq> 0" and "fr > 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   657
      and fr: "fp holomorphic_on cball z fr"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   658
              "\<And>w. w \<in> cball z fr - {z} \<Longrightarrow> f w = fp w * (w-z) powi fn \<and> fp w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   659
    using holomorphic_factor_puncture[OF f_iso f_ness f_nconst] by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   660
  have "f w \<noteq> 0" when " w \<noteq> z" "dist w z < fr" for w
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   661
  proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   662
    have "f w = fp w * (w-z) powi fn" "fp w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   663
      using fr that by (auto simp add: dist_commute)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   664
    moreover have "(w-z) powi fn \<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   665
      unfolding powr_eq_0_iff using \<open>w\<noteq>z\<close> by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   666
    ultimately show ?thesis by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   667
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   668
  then show ?thesis using \<open>fr>0\<close> unfolding eventually_at by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   669
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   670
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   671
lemma non_zero_neighbour_pole:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   672
  assumes "is_pole f z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   673
  shows "\<forall>\<^sub>F w in (at z). f w\<noteq>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   674
  using assms filterlim_at_infinity_imp_eventually_ne[of f "at z" 0]
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   675
  unfolding is_pole_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   676
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   677
lemma non_zero_neighbour_alt:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   678
  assumes holo: "f holomorphic_on S"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   679
      and "open S" "connected S" "z \<in> S"  "\<beta> \<in> S" "f \<beta> \<noteq> 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   680
    shows "\<forall>\<^sub>F w in (at z). f w\<noteq>0 \<and> w\<in>S"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   681
proof (cases "f z = 0")
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   682
  case True
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   683
  from isolated_zeros[OF holo \<open>open S\<close> \<open>connected S\<close> \<open>z \<in> S\<close> True \<open>\<beta> \<in> S\<close> \<open>f \<beta> \<noteq> 0\<close>]
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   684
  obtain r where "0 < r" "ball z r \<subseteq> S" "\<forall>w \<in> ball z r - {z}.f w \<noteq> 0" by metis
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   685
  then show ?thesis
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   686
    by (smt (verit) open_ball centre_in_ball eventually_at_topological insertE insert_Diff subsetD)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   687
next
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   688
  case False
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   689
  obtain r1 where r1: "r1>0" "\<forall>y. dist z y < r1 \<longrightarrow> f y \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   690
    using continuous_at_avoid[of z f, OF _ False] assms continuous_on_eq_continuous_at
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   691
      holo holomorphic_on_imp_continuous_on by blast
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   692
  obtain r2 where r2: "r2>0" "ball z r2 \<subseteq> S"
76895
498d8babe716 Further simplifications
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   693
    using assms openE by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   694
  show ?thesis unfolding eventually_at
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   695
    by (metis (no_types) dist_commute order.strict_trans linorder_less_linear mem_ball r1 r2 subsetD)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   696
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   697
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   698
lemma not_essential_times[singularity_intros]:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   699
  assumes f_ness: "not_essential f z" and g_ness: "not_essential g z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   700
  assumes f_iso: "isolated_singularity_at f z" and g_iso: "isolated_singularity_at g z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   701
  shows "not_essential (\<lambda>w. f w * g w) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   702
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   703
  define fg where "fg = (\<lambda>w. f w * g w)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   704
  have ?thesis when "\<not> ((\<exists>\<^sub>Fw in (at z). f w\<noteq>0) \<and> (\<exists>\<^sub>Fw in (at z). g w\<noteq>0))"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   705
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   706
    have "\<forall>\<^sub>Fw in (at z). fg w=0"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   707
      using fg_def frequently_elim1 not_eventually that by fastforce
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   708
    from tendsto_cong[OF this] have "fg \<midarrow>z\<rightarrow>0" by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   709
    then show ?thesis unfolding not_essential_def fg_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   710
  qed
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   711
  moreover have ?thesis when f_nconst: "\<exists>\<^sub>Fw in (at z). f w\<noteq>0" and g_nconst: "\<exists>\<^sub>Fw in (at z). g w\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   712
  proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   713
    obtain fn fp fr where [simp]: "fp z \<noteq> 0" and "fr > 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   714
          and fr: "fp holomorphic_on cball z fr"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   715
                  "\<forall>w\<in>cball z fr - {z}. f w = fp w * (w-z) powi fn \<and> fp w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   716
      using holomorphic_factor_puncture[OF f_iso f_ness f_nconst] by auto
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   717
    obtain gn gp gr where [simp]: "gp z \<noteq> 0" and "gr > 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   718
          and gr: "gp holomorphic_on cball z gr"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   719
                  "\<forall>w\<in>cball z gr - {z}. g w = gp w * (w-z) powi gn \<and> gp w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   720
      using holomorphic_factor_puncture[OF g_iso g_ness g_nconst] by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   721
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   722
    define r1 where "r1=(min fr gr)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   723
    have "r1>0" unfolding r1_def using  \<open>fr>0\<close> \<open>gr>0\<close> by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   724
    have fg_times: "fg w = (fp w * gp w) * (w-z) powi (fn+gn)" and fgp_nz: "fp w*gp w\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   725
      when "w\<in>ball z r1 - {z}" for w
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   726
    proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   727
      have "f w = fp w * (w-z) powi fn" "fp w\<noteq>0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   728
        using fr that unfolding r1_def by auto
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   729
      moreover have "g w = gp w * (w-z) powi gn" "gp w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   730
        using gr that unfolding r1_def by auto
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   731
      ultimately show "fg w = (fp w * gp w) * (w-z) powi (fn+gn)" "fp w*gp w\<noteq>0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   732
        using that by (auto simp add: fg_def power_int_add)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   733
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   734
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   735
    obtain [intro]: "fp \<midarrow>z\<rightarrow>fp z" "gp \<midarrow>z\<rightarrow>gp z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   736
        using fr(1) \<open>fr>0\<close> gr(1) \<open>gr>0\<close>
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   737
        by (metis centre_in_ball continuous_at continuous_on_interior
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   738
            holomorphic_on_imp_continuous_on interior_cball)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   739
    have ?thesis when "fn+gn>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   740
    proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   741
      have "(\<lambda>w. (fp w * gp w) * (w-z) ^ (nat (fn+gn))) \<midarrow>z\<rightarrow>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   742
        using that by (auto intro!:tendsto_eq_intros)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   743
      then have "fg \<midarrow>z\<rightarrow> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   744
        using Lim_transform_within[OF _ \<open>r1>0\<close>]
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   745
        by (smt (verit, best) Diff_iff dist_commute fg_times mem_ball power_int_def singletonD that zero_less_dist_iff)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   746
      then show ?thesis unfolding not_essential_def fg_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   747
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   748
    moreover have ?thesis when "fn+gn=0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   749
    proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   750
      have "(\<lambda>w. fp w * gp w) \<midarrow>z\<rightarrow>fp z*gp z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   751
        using that by (auto intro!:tendsto_eq_intros)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   752
      then have "fg \<midarrow>z\<rightarrow> fp z*gp z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   753
        apply (elim Lim_transform_within[OF _ \<open>r1>0\<close>])
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   754
        apply (subst fg_times)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   755
        by (auto simp add: dist_commute that)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   756
      then show ?thesis unfolding not_essential_def fg_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   757
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   758
    moreover have ?thesis when "fn+gn<0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   759
    proof -
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   760
      have "LIM x at z. (x - z) ^ nat (- (fn + gn)) :> at 0"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   761
        using eventually_at_topological that
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   762
        by (force intro!: tendsto_eq_intros filterlim_atI)
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   763
      moreover have "\<exists>c. (\<lambda>c. fp c * gp c) \<midarrow>z\<rightarrow> c \<and> 0 \<noteq> c"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   764
        using \<open>fp \<midarrow>z\<rightarrow> fp z\<close> \<open>gp \<midarrow>z\<rightarrow> gp z\<close> tendsto_mult by fastforce
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   765
      ultimately have "LIM w (at z). fp w * gp w / (w-z)^nat (-(fn+gn)) :> at_infinity"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   766
        using filterlim_divide_at_infinity by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   767
      then have "is_pole fg z" unfolding is_pole_def
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   768
        apply (elim filterlim_transform_within[OF _ _ \<open>r1>0\<close>])
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   769
        using that
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
   770
        by (simp_all add: dist_commute fg_times of_int_of_nat divide_simps power_int_def del: minus_add_distrib)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   771
      then show ?thesis unfolding not_essential_def fg_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   772
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   773
    ultimately show ?thesis unfolding not_essential_def fg_def by fastforce
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   774
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   775
  ultimately show ?thesis by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   776
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   777
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   778
lemma not_essential_inverse[singularity_intros]:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   779
  assumes f_ness: "not_essential f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   780
  assumes f_iso: "isolated_singularity_at f z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   781
  shows "not_essential (\<lambda>w. inverse (f w)) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   782
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   783
  define vf where "vf = (\<lambda>w. inverse (f w))"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   784
  have ?thesis when "\<not>(\<exists>\<^sub>Fw in (at z). f w\<noteq>0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   785
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   786
    have "\<forall>\<^sub>Fw in (at z). f w=0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   787
      using not_eventually that by fastforce
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   788
    then have "vf \<midarrow>z\<rightarrow>0" 
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   789
      unfolding vf_def by (simp add: tendsto_eventually)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   790
    then show ?thesis 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   791
      unfolding not_essential_def vf_def by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   792
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   793
  moreover have ?thesis when "is_pole f z"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   794
    by (metis (mono_tags, lifting) filterlim_at filterlim_inverse_at_iff is_pole_def
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   795
        not_essential_def that)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   796
  moreover have ?thesis when "\<exists>x. f\<midarrow>z\<rightarrow>x " and f_nconst: "\<exists>\<^sub>Fw in (at z). f w\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   797
  proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   798
    from that obtain fz where fz: "f\<midarrow>z\<rightarrow>fz" by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   799
    have ?thesis when "fz=0"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   800
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   801
    proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   802
      have "(\<lambda>w. inverse (vf w)) \<midarrow>z\<rightarrow>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   803
        using fz that unfolding vf_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   804
      moreover have "\<forall>\<^sub>F w in at z. inverse (vf w) \<noteq> 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   805
        using non_zero_neighbour[OF f_iso f_ness f_nconst]
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   806
        unfolding vf_def by auto
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   807
      ultimately show ?thesis unfolding not_essential_def vf_def
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   808
         using filterlim_atI filterlim_inverse_at_iff is_pole_def by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   809
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   810
    moreover have ?thesis when "fz\<noteq>0"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   811
      using fz not_essential_def tendsto_inverse that by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   812
    ultimately show ?thesis by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   813
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   814
  ultimately show ?thesis using f_ness unfolding not_essential_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   815
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   816
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   817
lemma isolated_singularity_at_inverse[singularity_intros]:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   818
  assumes f_iso: "isolated_singularity_at f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   819
      and f_ness: "not_essential f z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   820
  shows "isolated_singularity_at (\<lambda>w. inverse (f w)) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   821
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   822
  define vf where "vf = (\<lambda>w. inverse (f w))"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   823
  have ?thesis when "\<not>(\<exists>\<^sub>Fw in (at z). f w\<noteq>0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   824
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   825
    have "\<forall>\<^sub>Fw in (at z). f w=0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   826
      using that[unfolded frequently_def, simplified] by (auto elim: eventually_rev_mp)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   827
    then have "\<forall>\<^sub>Fw in (at z). vf w=0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   828
      unfolding vf_def by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   829
    then obtain d1 where "d1>0" and d1: "\<forall>x. x \<noteq> z \<and> dist x z < d1 \<longrightarrow> vf x = 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   830
      unfolding eventually_at by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   831
    then have "vf holomorphic_on ball z d1-{z}"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   832
      using holomorphic_transform[of "\<lambda>_. 0"]
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   833
      by (metis Diff_iff dist_commute holomorphic_on_const insert_iff mem_ball)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   834
    then have "vf analytic_on ball z d1 - {z}"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   835
      by (simp add: analytic_on_open open_delete)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   836
    then show ?thesis 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   837
      using \<open>d1>0\<close> unfolding isolated_singularity_at_def vf_def by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   838
  qed
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   839
  moreover have ?thesis when f_nconst: "\<exists>\<^sub>Fw in (at z). f w\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   840
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   841
    have "\<forall>\<^sub>F w in at z. f w \<noteq> 0" using non_zero_neighbour[OF f_iso f_ness f_nconst] .
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   842
    then obtain d1 where d1: "d1>0" "\<forall>x. x \<noteq> z \<and> dist x z < d1 \<longrightarrow> f x \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   843
      unfolding eventually_at by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   844
    obtain d2 where "d2>0" and d2: "f analytic_on ball z d2 - {z}"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   845
      using f_iso unfolding isolated_singularity_at_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   846
    define d3 where "d3=min d1 d2"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   847
    have "d3>0" unfolding d3_def using \<open>d1>0\<close> \<open>d2>0\<close> by auto
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   848
    moreover
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   849
    have "f analytic_on ball z d3 - {z}"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   850
      by (smt (verit, best) Diff_iff analytic_on_analytic_at d2 d3_def mem_ball)
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   851
    then have "vf analytic_on ball z d3 - {z}"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   852
      unfolding vf_def
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   853
      by (intro analytic_on_inverse; simp add: d1(2) d3_def dist_commute)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   854
    ultimately show ?thesis 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   855
      unfolding isolated_singularity_at_def vf_def by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   856
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   857
  ultimately show ?thesis by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   858
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   859
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   860
lemma not_essential_divide[singularity_intros]:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   861
  assumes f_ness: "not_essential f z" and g_ness: "not_essential g z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   862
  assumes f_iso: "isolated_singularity_at f z" and g_iso: "isolated_singularity_at g z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   863
  shows "not_essential (\<lambda>w. f w / g w) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   864
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   865
  have "not_essential (\<lambda>w. f w * inverse (g w)) z"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   866
    by (simp add: f_iso f_ness g_iso g_ness isolated_singularity_at_inverse
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   867
        not_essential_inverse not_essential_times)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   868
  then show ?thesis by (simp add: field_simps)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   869
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   870
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   871
lemma
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   872
  assumes f_iso: "isolated_singularity_at f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   873
      and g_iso: "isolated_singularity_at g z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   874
    shows isolated_singularity_at_times[singularity_intros]:
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   875
              "isolated_singularity_at (\<lambda>w. f w * g w) z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   876
      and isolated_singularity_at_add[singularity_intros]:
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   877
              "isolated_singularity_at (\<lambda>w. f w + g w) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   878
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   879
  obtain d1 d2 where "d1>0" "d2>0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   880
      and d1: "f analytic_on ball z d1 - {z}" and d2: "g analytic_on ball z d2 - {z}"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   881
    using f_iso g_iso unfolding isolated_singularity_at_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   882
  define d3 where "d3=min d1 d2"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   883
  have "d3>0" unfolding d3_def using \<open>d1>0\<close> \<open>d2>0\<close> by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   884
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   885
  have fan: "f analytic_on ball z d3 - {z}"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   886
    by (smt (verit, best) Diff_iff analytic_on_analytic_at d1 d3_def mem_ball)
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   887
  have gan: "g analytic_on ball z d3 - {z}"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   888
    by (smt (verit, best) Diff_iff analytic_on_analytic_at d2 d3_def mem_ball)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   889
  have "(\<lambda>w. f w * g w) analytic_on ball z d3 - {z}"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   890
    using analytic_on_mult fan gan by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   891
  then show "isolated_singularity_at (\<lambda>w. f w * g w) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   892
    using \<open>d3>0\<close> unfolding isolated_singularity_at_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   893
  have "(\<lambda>w. f w + g w) analytic_on ball z d3 - {z}"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
   894
    using analytic_on_add fan gan by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   895
  then show "isolated_singularity_at (\<lambda>w. f w + g w) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   896
    using \<open>d3>0\<close> unfolding isolated_singularity_at_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   897
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   898
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   899
lemma isolated_singularity_at_uminus[singularity_intros]:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
   900
  assumes f_iso: "isolated_singularity_at f z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   901
  shows "isolated_singularity_at (\<lambda>w. - f w) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   902
  using assms unfolding isolated_singularity_at_def using analytic_on_neg by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   903
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   904
lemma isolated_singularity_at_id[singularity_intros]:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   905
     "isolated_singularity_at (\<lambda>w. w) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   906
  unfolding isolated_singularity_at_def by (simp add: gt_ex)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   907
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   908
lemma isolated_singularity_at_minus[singularity_intros]:
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   909
  assumes "isolated_singularity_at f z" and "isolated_singularity_at g z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   910
  shows "isolated_singularity_at (\<lambda>w. f w - g w) z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   911
  unfolding diff_conv_add_uminus
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   912
  using assms isolated_singularity_at_add isolated_singularity_at_uminus by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   913
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   914
lemma isolated_singularity_at_divide[singularity_intros]:
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   915
  assumes "isolated_singularity_at f z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   916
      and "isolated_singularity_at g z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   917
      and "not_essential g z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   918
    shows "isolated_singularity_at (\<lambda>w. f w / g w) z"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   919
  unfolding divide_inverse
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
   920
  by (simp add: assms isolated_singularity_at_inverse isolated_singularity_at_times)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   921
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   922
lemma isolated_singularity_at_const[singularity_intros]:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   923
    "isolated_singularity_at (\<lambda>w. c) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   924
  unfolding isolated_singularity_at_def by (simp add: gt_ex)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   925
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   926
lemma isolated_singularity_at_holomorphic:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   927
  assumes "f holomorphic_on s-{z}" "open s" "z\<in>s"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   928
  shows "isolated_singularity_at f z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   929
  using assms unfolding isolated_singularity_at_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   930
  by (metis analytic_on_holomorphic centre_in_ball insert_Diff openE open_delete subset_insert_iff)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
   931
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   932
lemma isolated_singularity_at_altdef:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   933
  "isolated_singularity_at f z \<longleftrightarrow> eventually (\<lambda>z. f analytic_on {z}) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   934
proof
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   935
  assume "isolated_singularity_at f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   936
  then obtain r where r: "r > 0" "f analytic_on ball z r - {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   937
    unfolding isolated_singularity_at_def by blast
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   938
  have "eventually (\<lambda>w. w \<in> ball z r - {z}) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   939
    using r(1) by (intro eventually_at_in_open) auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   940
  thus "eventually (\<lambda>z. f analytic_on {z}) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   941
    by eventually_elim (use r analytic_on_subset in auto)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   942
next
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   943
  assume "eventually (\<lambda>z. f analytic_on {z}) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   944
  then obtain A where A: "open A" "z \<in> A" "\<And>w. w \<in> A - {z} \<Longrightarrow> f analytic_on {w}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   945
    unfolding eventually_at_topological by blast
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   946
  then show "isolated_singularity_at f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   947
    by (meson analytic_imp_holomorphic analytic_on_analytic_at isolated_singularity_at_holomorphic)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   948
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
   949
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   950
lemma isolated_singularity_at_shift:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   951
  assumes "isolated_singularity_at (\<lambda>x. f (x + w)) z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   952
  shows   "isolated_singularity_at f (z + w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   953
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   954
  from assms obtain r where r: "r > 0" and ana: "(\<lambda>x. f (x + w)) analytic_on ball z r - {z}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   955
    unfolding isolated_singularity_at_def by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   956
  have "((\<lambda>x. f (x + w)) \<circ> (\<lambda>x. x - w)) analytic_on (ball (z + w) r - {z + w})"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   957
    by (rule analytic_on_compose_gen[OF _ ana])
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   958
       (auto simp: dist_norm algebra_simps intro!: analytic_intros)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   959
  hence "f analytic_on (ball (z + w) r - {z + w})"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   960
    by (simp add: o_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   961
  thus ?thesis using r
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   962
    unfolding isolated_singularity_at_def by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   963
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   964
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   965
lemma isolated_singularity_at_shift_iff:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   966
  "isolated_singularity_at f (z + w) \<longleftrightarrow> isolated_singularity_at (\<lambda>x. f (x + w)) z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   967
  using isolated_singularity_at_shift[of f w z]
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   968
        isolated_singularity_at_shift[of "\<lambda>x. f (x + w)" "-w" "w + z"]
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   969
  by (auto simp: algebra_simps)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   970
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   971
lemma isolated_singularity_at_shift_0:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   972
  "NO_MATCH 0 z \<Longrightarrow> isolated_singularity_at f z \<longleftrightarrow> isolated_singularity_at (\<lambda>x. f (z + x)) 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   973
  using isolated_singularity_at_shift_iff[of f 0 z] by (simp add: add_ac)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   974
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   975
lemma not_essential_shift:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   976
  assumes "not_essential (\<lambda>x. f (x + w)) z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   977
  shows   "not_essential f (z + w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   978
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   979
  from assms consider c where "(\<lambda>x. f (x + w)) \<midarrow>z\<rightarrow> c" | "is_pole (\<lambda>x. f (x + w)) z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   980
    unfolding not_essential_def by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   981
  thus ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   982
  proof cases
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   983
    case (1 c)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   984
    hence "f \<midarrow>z + w\<rightarrow> c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   985
      by (smt (verit, ccfv_SIG) LIM_cong add.assoc filterlim_at_to_0)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   986
    thus ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   987
      by (auto simp: not_essential_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   988
  next
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   989
    case 2
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   990
    hence "is_pole f (z + w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   991
      by (subst is_pole_shift_iff [symmetric]) (auto simp: o_def add_ac)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   992
    thus ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   993
      by (auto simp: not_essential_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   994
  qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   995
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   996
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   997
lemma not_essential_shift_iff: "not_essential f (z + w) \<longleftrightarrow> not_essential (\<lambda>x. f (x + w)) z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   998
  using not_essential_shift[of f w z]
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
   999
        not_essential_shift[of "\<lambda>x. f (x + w)" "-w" "w + z"]
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1000
  by (auto simp: algebra_simps)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1001
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1002
lemma not_essential_shift_0:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1003
  "NO_MATCH 0 z \<Longrightarrow> not_essential f z \<longleftrightarrow> not_essential (\<lambda>x. f (z + x)) 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1004
  using not_essential_shift_iff[of f 0 z] by (simp add: add_ac)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1005
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1006
lemma not_essential_holomorphic:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1007
  assumes "f holomorphic_on A" "x \<in> A" "open A"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1008
  shows   "not_essential f x"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1009
  by (metis assms at_within_open continuous_on holomorphic_on_imp_continuous_on not_essential_def)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1010
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1011
lemma not_essential_analytic:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1012
  assumes "f analytic_on {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1013
  shows   "not_essential f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1014
  using analytic_at assms not_essential_holomorphic by blast
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1015
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1016
lemma not_essential_id [singularity_intros]: "not_essential (\<lambda>w. w) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1017
  by (simp add: not_essential_analytic)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1018
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1019
lemma is_pole_imp_not_essential [intro]: "is_pole f z \<Longrightarrow> not_essential f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1020
  by (auto simp: not_essential_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1021
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1022
lemma tendsto_imp_not_essential [intro]: "f \<midarrow>z\<rightarrow> c \<Longrightarrow> not_essential f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1023
  by (auto simp: not_essential_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1024
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1025
lemma eventually_not_pole:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1026
  assumes "isolated_singularity_at f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1027
  shows   "eventually (\<lambda>w. \<not>is_pole f w) (at z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1028
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1029
  from assms obtain r where "r > 0" and r: "f analytic_on ball z r - {z}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1030
    by (auto simp: isolated_singularity_at_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1031
  then have "eventually (\<lambda>w. w \<in> ball z r - {z}) (at z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1032
    by (intro eventually_at_in_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1033
  thus "eventually (\<lambda>w. \<not>is_pole f w) (at z)"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1034
    by (metis (no_types, lifting) analytic_at analytic_on_analytic_at eventually_mono not_is_pole_holomorphic r)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1035
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1036
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1037
lemma not_islimpt_poles:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1038
  assumes "isolated_singularity_at f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1039
  shows   "\<not>z islimpt {w. is_pole f w}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1040
  using eventually_not_pole [OF assms]
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1041
  by (auto simp: islimpt_conv_frequently_at frequently_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1042
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1043
lemma analytic_at_imp_no_pole: "f analytic_on {z} \<Longrightarrow> \<not>is_pole f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1044
  using analytic_at not_is_pole_holomorphic by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1045
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1046
lemma not_essential_const [singularity_intros]: "not_essential (\<lambda>_. c) z"
77277
c6b50597abbc More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents: 77228
diff changeset
  1047
  by blast
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1048
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1049
lemma not_essential_uminus [singularity_intros]:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1050
  assumes f_ness: "not_essential f z"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1051
  assumes f_iso: "isolated_singularity_at f z"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1052
  shows "not_essential (\<lambda>w. -f w) z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1053
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1054
  have "not_essential (\<lambda>w. -1 * f w) z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1055
    by (intro assms singularity_intros)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1056
  thus ?thesis by simp
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1057
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1058
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1059
lemma isolated_singularity_at_analytic:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1060
  assumes "f analytic_on {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1061
  shows   "isolated_singularity_at f z"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1062
  by (meson Diff_subset analytic_at assms holomorphic_on_subset isolated_singularity_at_holomorphic)
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1063
82310
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1064
lemma isolated_singularity_sum [singularity_intros]:
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1065
  assumes "\<And>x. x \<in> A \<Longrightarrow> isolated_singularity_at (f x) z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1066
  shows   "isolated_singularity_at (\<lambda>w. \<Sum>x\<in>A. f x w) z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1067
  using assms by (induction A rule: infinite_finite_induct) (auto intro!: singularity_intros)
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1068
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1069
lemma isolated_singularity_prod [singularity_intros]:
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1070
  assumes "\<And>x. x \<in> A \<Longrightarrow> isolated_singularity_at (f x) z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1071
  shows   "isolated_singularity_at (\<lambda>w. \<Prod>x\<in>A. f x w) z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1072
  using assms by (induction A rule: infinite_finite_induct) (auto intro!: singularity_intros)
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1073
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1074
lemma isolated_singularity_sum_list [singularity_intros]:
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1075
  assumes "\<And>f. f \<in> set fs \<Longrightarrow> isolated_singularity_at f z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1076
  shows   "isolated_singularity_at (\<lambda>w. \<Sum>f\<leftarrow>fs. f w) z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1077
  using assms by (induction fs) (auto intro!: singularity_intros)
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1078
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1079
lemma isolated_singularity_prod_list [singularity_intros]:
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1080
  assumes "\<And>f. f \<in> set fs \<Longrightarrow> isolated_singularity_at f z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1081
  shows   "isolated_singularity_at (\<lambda>w. \<Prod>f\<leftarrow>fs. f w) z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1082
  using assms by (induction fs) (auto intro!: singularity_intros)
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1083
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1084
lemma isolated_singularity_sum_mset [singularity_intros]:
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1085
  assumes "\<And>f. f \<in># F \<Longrightarrow> isolated_singularity_at f z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1086
  shows   "isolated_singularity_at (\<lambda>w. \<Sum>f\<in>#F. f w) z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1087
  using assms by (induction F) (auto intro!: singularity_intros)
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1088
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1089
lemma isolated_singularity_prod_mset [singularity_intros]:
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1090
  assumes "\<And>f. f \<in># F \<Longrightarrow> isolated_singularity_at f z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1091
  shows   "isolated_singularity_at (\<lambda>w. \<Prod>f\<in>#F. f w) z"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1092
  using assms by (induction F) (auto intro!: singularity_intros)
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1093
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1094
lemma analytic_nhd_imp_isolated_singularity:
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1095
  assumes "f analytic_on A - {x}" "x \<in> A" "open A"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1096
  shows   "isolated_singularity_at f x"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1097
  unfolding isolated_singularity_at_def using assms
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1098
  using analytic_imp_holomorphic isolated_singularity_at_def isolated_singularity_at_holomorphic by blast
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1099
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1100
lemma isolated_singularity_at_iff_analytic_nhd:
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1101
  "isolated_singularity_at f x \<longleftrightarrow> (\<exists>A. x \<in> A \<and> open A \<and> f analytic_on A - {x})"
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1102
  by (meson open_ball analytic_nhd_imp_isolated_singularity
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1103
            centre_in_ball isolated_singularity_at_def)
41f5266e5595 New theorems, mostly from the number theory project
paulson <lp15@cam.ac.uk>
parents: 81899
diff changeset
  1104
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1105
subsection \<open>The order of non-essential singularities (i.e. removable singularities or poles)\<close>
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1106
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1107
definition\<^marker>\<open>tag important\<close> zorder :: "(complex \<Rightarrow> complex) \<Rightarrow> complex \<Rightarrow> int" where
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1108
  "zorder f z = (THE n. (\<exists>h r. r>0 \<and> h holomorphic_on cball z r \<and> h z\<noteq>0
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1109
                   \<and> (\<forall>w\<in>cball z r - {z}. f w =  h w * (w-z) powi n
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1110
                   \<and> h w \<noteq>0)))"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1111
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1112
definition\<^marker>\<open>tag important\<close> zor_poly
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1113
    :: "[complex \<Rightarrow> complex, complex] \<Rightarrow> complex \<Rightarrow> complex" where
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1114
  "zor_poly f z = (SOME h. \<exists>r. r > 0 \<and> h holomorphic_on cball z r \<and> h z \<noteq> 0
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1115
                   \<and> (\<forall>w\<in>cball z r - {z}. f w =  h w * (w-z) powi (zorder f z)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1116
                   \<and> h w \<noteq>0))"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1117
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1118
lemma zorder_exist:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1119
  fixes f:: "complex \<Rightarrow> complex" and z::complex
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1120
  defines "n \<equiv> zorder f z" and "g \<equiv> zor_poly f z"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1121
  assumes f_iso: "isolated_singularity_at f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1122
      and f_ness: "not_essential f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1123
      and f_nconst: "\<exists>\<^sub>Fw in (at z). f w\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1124
  shows "g z\<noteq>0 \<and> (\<exists>r. r>0 \<and> g holomorphic_on cball z r
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1125
    \<and> (\<forall>w\<in>cball z r - {z}. f w  = g w * (w-z) powi n  \<and> g w \<noteq>0))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1126
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1127
  define P where "P = (\<lambda>n g r. 0 < r \<and> g holomorphic_on cball z r \<and> g z\<noteq>0
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1128
          \<and> (\<forall>w\<in>cball z r - {z}. f w = g w * (w-z) powi n \<and> g w\<noteq>0))"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1129
  have "\<exists>!k. \<exists>g r. P k g r"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1130
    using holomorphic_factor_puncture[OF assms(3-)] unfolding P_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1131
  then have "\<exists>g r. P n g r"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1132
    unfolding n_def P_def zorder_def by (rule theI')
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1133
  then have "\<exists>r. P n g r"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1134
    unfolding P_def zor_poly_def g_def n_def by (rule someI_ex)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1135
  then obtain r1 where "P n g r1" 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1136
    by auto
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1137
  then show ?thesis 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1138
    unfolding P_def by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1139
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1140
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1141
lemma zorder_shift:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1142
  shows  "zorder f z = zorder (\<lambda>u. f (u + z)) 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1143
  unfolding zorder_def
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1144
  apply (rule arg_cong [of concl: The])
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1145
  apply (auto simp: fun_eq_iff Ball_def dist_norm)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1146
  subgoal for x h r
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1147
    apply (rule_tac x="h o (+)z" in exI)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1148
    apply (rule_tac x="r" in exI)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1149
    apply (intro conjI holomorphic_on_compose holomorphic_intros)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1150
       apply (simp_all flip: cball_translation)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1151
    apply (simp add: add.commute)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1152
    done
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1153
  subgoal for x h r
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1154
    apply (rule_tac x="h o (\<lambda>u. u-z)" in exI)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1155
    apply (rule_tac x="r" in exI)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1156
    apply (intro conjI holomorphic_on_compose holomorphic_intros)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1157
       apply (simp_all flip: cball_translation_subtract)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1158
    by (metis diff_add_cancel eq_iff_diff_eq_0 norm_minus_commute)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1159
  done
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1160
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1161
lemma zorder_shift': "NO_MATCH 0 z \<Longrightarrow> zorder f z = zorder (\<lambda>u. f (u + z)) 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1162
  by (rule zorder_shift)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1163
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1164
lemma
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1165
  fixes f:: "complex \<Rightarrow> complex" and z::complex
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1166
  assumes f_iso: "isolated_singularity_at f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1167
      and f_ness: "not_essential f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1168
      and f_nconst: "\<exists>\<^sub>Fw in (at z). f w\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1169
    shows zorder_inverse: "zorder (\<lambda>w. inverse (f w)) z = - zorder f z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1170
      and zor_poly_inverse: "\<forall>\<^sub>Fw in (at z). zor_poly (\<lambda>w. inverse (f w)) z w
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1171
                                                = inverse (zor_poly f z w)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1172
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1173
  define vf where "vf = (\<lambda>w. inverse (f w))"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1174
  define fn vfn where
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1175
    "fn = zorder f z"  and "vfn = zorder vf z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1176
  define fp vfp where
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1177
    "fp = zor_poly f z" and "vfp = zor_poly vf z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1178
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1179
  obtain fr where [simp]: "fp z \<noteq> 0" and "fr > 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1180
          and fr: "fp holomorphic_on cball z fr"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1181
                  "\<forall>w\<in>cball z fr - {z}. f w = fp w * (w-z) powi fn \<and> fp w \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1182
    using zorder_exist[OF f_iso f_ness f_nconst,folded fn_def fp_def]
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1183
    by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1184
  have fr_inverse: "vf w = (inverse (fp w)) * (w-z) powi (-fn)"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1185
        and fr_nz: "inverse (fp w) \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1186
    when "w\<in>ball z fr - {z}" for w
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1187
  proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1188
    have "f w = fp w * (w-z) powi fn" "fp w \<noteq> 0"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1189
      using fr(2) that by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1190
    then show "vf w = (inverse (fp w)) * (w-z) powi (-fn)" "inverse (fp w)\<noteq>0"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1191
      by (simp_all add: power_int_minus vf_def)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1192
  qed
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1193
  obtain vfr where [simp]: "vfp z \<noteq> 0" and "vfr>0" and vfr: "vfp holomorphic_on cball z vfr"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1194
      "(\<forall>w\<in>cball z vfr - {z}. vf w = vfp w * (w-z) powi vfn \<and> vfp w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1195
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1196
    have "isolated_singularity_at vf z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1197
      using isolated_singularity_at_inverse[OF f_iso f_ness] unfolding vf_def .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1198
    moreover have "not_essential vf z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1199
      using not_essential_inverse[OF f_ness f_iso] unfolding vf_def .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1200
    moreover have "\<exists>\<^sub>F w in at z. vf w \<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1201
      using f_nconst unfolding vf_def by (auto elim: frequently_elim1)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1202
    ultimately show ?thesis using zorder_exist[of vf z, folded vfn_def vfp_def] that by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1203
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1204
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1205
  define r1 where "r1 = min fr vfr"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1206
  have "r1>0" using \<open>fr>0\<close> \<open>vfr>0\<close> unfolding r1_def by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1207
  show "vfn = - fn"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1208
  proof (rule holomorphic_factor_unique)
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1209
    have \<section>: "\<And>w. \<lbrakk>fp w = 0; dist z w < fr\<rbrakk> \<Longrightarrow> False"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1210
      using fr_nz by force
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1211
    then show "\<forall>w\<in>ball z r1 - {z}.
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1212
               vf w = vfp w * (w-z) powi vfn \<and>
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1213
               vfp w \<noteq> 0 \<and> vf w = inverse (fp w) * (w-z) powi (- fn) \<and>
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1214
               inverse (fp w) \<noteq> 0"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1215
      using fr_inverse r1_def vfr(2)
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1216
      by (smt (verit) Diff_iff inverse_nonzero_iff_nonzero mem_ball mem_cball)
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1217
    show "vfp holomorphic_on ball z r1"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1218
      using r1_def vfr(1) by auto
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1219
    show "(\<lambda>w. inverse (fp w)) holomorphic_on ball z r1"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1220
      by (metis \<section> ball_subset_cball fr(1) holomorphic_on_inverse holomorphic_on_subset mem_ball min.cobounded2 min.commute r1_def subset_ball)
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1221
  qed (use \<open>r1>0\<close> in auto)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1222
  have "vfp w = inverse (fp w)" when "w\<in>ball z r1-{z}" for w
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1223
  proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1224
    have "w \<in> ball z fr - {z}" "w \<in> cball z vfr - {z}"  "w\<noteq>z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1225
      using that unfolding r1_def by auto
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1226
    then show ?thesis
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1227
      by (metis \<open>vfn = - fn\<close> power_int_not_zero right_minus_eq  fr_inverse vfr(2)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1228
          vector_space_over_itself.scale_right_imp_eq) 
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1229
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1230
  then show "\<forall>\<^sub>Fw in (at z). vfp w = inverse (fp w)"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1231
    unfolding eventually_at by (metis DiffI dist_commute mem_ball singletonD \<open>r1>0\<close>)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1232
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1233
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1234
lemma zor_poly_shift:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1235
  assumes iso1: "isolated_singularity_at f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1236
    and ness1: "not_essential f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1237
    and nzero1: "\<exists>\<^sub>F w in at z. f w \<noteq> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1238
  shows "\<forall>\<^sub>F w in nhds z. zor_poly f z w = zor_poly (\<lambda>u. f (z + u)) 0 (w-z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1239
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1240
  obtain r1 where "r1>0" "zor_poly f z z \<noteq> 0" and
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1241
      holo1: "zor_poly f z holomorphic_on cball z r1" and
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1242
      rball1: "\<forall>w\<in>cball z r1 - {z}.
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1243
           f w = zor_poly f z w * (w-z) powi (zorder f z) \<and>
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1244
           zor_poly f z w \<noteq> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1245
    using zorder_exist[OF iso1 ness1 nzero1] by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1246
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1247
  define ff where "ff=(\<lambda>u. f (z + u))"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1248
  have "isolated_singularity_at ff 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1249
    unfolding ff_def
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1250
    using iso1 isolated_singularity_at_shift_iff[of f 0 z]
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1251
    by (simp add: algebra_simps)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1252
  moreover have "not_essential ff 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1253
    unfolding ff_def
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1254
    using ness1 not_essential_shift_iff[of f 0 z]
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1255
    by (simp add: algebra_simps)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1256
  moreover have "\<exists>\<^sub>F w in at 0. ff w \<noteq> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1257
    unfolding ff_def using nzero1
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1258
    by (smt (verit, ccfv_SIG) add.commute eventually_at_to_0
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1259
        eventually_mono not_frequently)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1260
  ultimately 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1261
  obtain r2 where "r2>0" "zor_poly ff 0 0 \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1262
          and holo2: "zor_poly ff 0 holomorphic_on cball 0 r2" 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1263
          and rball2: "\<forall>w\<in>cball 0 r2 - {0}.
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1264
               ff w = zor_poly ff 0 w * w powi (zorder ff 0) \<and> zor_poly ff 0 w \<noteq> 0"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1265
    using zorder_exist[of ff 0] by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1266
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1267
  define r where "r=min r1 r2"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1268
  have "r>0" using \<open>r1>0\<close> \<open>r2>0\<close> unfolding r_def by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1269
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1270
  have "zor_poly f z w = zor_poly ff 0 (w-z)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1271
    if "w\<in>ball z r - {z}" for w
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1272
  proof -
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1273
    define n where "n \<equiv> zorder f z"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1274
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1275
    have "f w = zor_poly f z w * (w-z) powi n"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1276
      using n_def r_def rball1 that by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1277
    moreover have "f w = zor_poly ff 0 (w-z) * (w-z) powi n"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1278
    proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1279
      have "w-z\<in>cball 0 r2 - {0}"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1280
        using r_def that by (auto simp: dist_complex_def)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1281
      then have "ff (w-z) = zor_poly ff 0 (w-z) * (w-z) powi (zorder ff 0)"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1282
        using rball2 by blast
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1283
      moreover have "of_int (zorder ff 0) = n"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1284
        unfolding n_def ff_def by (simp add:zorder_shift' add.commute)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1285
      ultimately show ?thesis unfolding ff_def by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1286
    qed
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1287
    ultimately have "zor_poly f z w * (w-z) powi n = zor_poly ff 0 (w-z) * (w-z) powi n"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1288
      by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1289
    moreover have "(w-z) powi n \<noteq>0"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1290
      using that by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1291
    ultimately show ?thesis
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1292
      using mult_cancel_right by blast
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1293
  qed
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1294
  then have "\<forall>\<^sub>F w in at z. zor_poly f z w = zor_poly ff 0 (w-z)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1295
    unfolding eventually_at
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1296
    by (metis DiffI \<open>0 < r\<close> dist_commute mem_ball singletonD)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1297
  moreover have "isCont (zor_poly f z) z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1298
    using holo1[THEN holomorphic_on_imp_continuous_on]
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1299
    by (simp add: \<open>0 < r1\<close> continuous_on_interior)
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1300
  moreover 
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1301
  have "isCont (zor_poly ff 0) 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1302
    using \<open>0 < r2\<close> continuous_on_interior holo2 holomorphic_on_imp_continuous_on
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1303
    by fastforce
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1304
  then have "isCont (\<lambda>w. zor_poly ff 0 (w-z)) z"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1305
      unfolding isCont_iff by simp
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1306
  ultimately show "\<forall>\<^sub>F w in nhds z. zor_poly f z w = zor_poly ff 0 (w-z)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1307
    by (elim at_within_isCont_imp_nhds;auto)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1308
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1309
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1310
lemma
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1311
  fixes f g:: "complex \<Rightarrow> complex" and z::complex
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1312
  assumes f_iso: "isolated_singularity_at f z" and g_iso: "isolated_singularity_at g z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1313
      and f_ness: "not_essential f z" and g_ness: "not_essential g z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1314
      and fg_nconst: "\<exists>\<^sub>Fw in (at z). f w * g w\<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1315
  shows zorder_times: "zorder (\<lambda>w. f w * g w) z = zorder f z + zorder g z" and
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1316
        zor_poly_times: "\<forall>\<^sub>Fw in (at z). zor_poly (\<lambda>w. f w * g w) z w
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1317
                                                  = zor_poly f z w *zor_poly g z w"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1318
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1319
  define fg where "fg = (\<lambda>w. f w * g w)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1320
  define fn gn fgn where
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1321
    "fn = zorder f z" and "gn = zorder g z" and "fgn = zorder fg z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1322
  define fp gp fgp where
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1323
    "fp = zor_poly f z" and "gp = zor_poly g z" and "fgp = zor_poly fg z"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1324
  have f_nconst: "\<exists>\<^sub>Fw in (at z). f w \<noteq> 0" and g_nconst: "\<exists>\<^sub>Fw in (at z).g w\<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1325
    using fg_nconst by (auto elim!:frequently_elim1)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1326
  obtain fr where [simp]: "fp z \<noteq> 0" and "fr > 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1327
          and fr: "fp holomorphic_on cball z fr"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1328
                  "\<forall>w\<in>cball z fr - {z}. f w = fp w * (w-z) powi fn \<and> fp w \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1329
    using zorder_exist[OF f_iso f_ness f_nconst,folded fp_def fn_def] by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1330
  obtain gr where [simp]: "gp z \<noteq> 0" and "gr > 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1331
          and gr: "gp holomorphic_on cball z gr"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1332
                  "\<forall>w\<in>cball z gr - {z}. g w = gp w * (w-z) powi gn \<and> gp w \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1333
    using zorder_exist[OF g_iso g_ness g_nconst,folded gn_def gp_def] by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1334
  define r1 where "r1=min fr gr"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1335
  have "r1>0" unfolding r1_def using \<open>fr>0\<close> \<open>gr>0\<close> by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1336
  have fg_times: "fg w = (fp w * gp w) * (w-z) powi (fn+gn)" and fgp_nz: "fp w*gp w\<noteq>0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1337
    when "w\<in>ball z r1 - {z}" for w
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1338
  proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1339
    have "f w = fp w * (w-z) powi fn" "fp w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1340
      using fr(2) r1_def that by auto
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1341
    moreover have "g w = gp w * (w-z) powi gn" "gp w \<noteq> 0"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1342
      using gr(2) that unfolding r1_def by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1343
    ultimately show "fg w = (fp w * gp w) * (w-z) powi (fn+gn)" "fp w*gp w\<noteq>0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1344
      using that unfolding fg_def by (auto simp add: power_int_add)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1345
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1346
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1347
  obtain fgr where [simp]: "fgp z \<noteq> 0" and "fgr > 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1348
          and fgr: "fgp holomorphic_on cball z fgr"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1349
                   "\<forall>w\<in>cball z fgr - {z}. fg w = fgp w * (w-z) powi fgn \<and> fgp w \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1350
  proof -
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1351
    have "isolated_singularity_at fg z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1352
      unfolding fg_def using isolated_singularity_at_times[OF f_iso g_iso] .
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1353
    moreover have "not_essential fg z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1354
      by (simp add: f_iso f_ness fg_def g_iso g_ness not_essential_times)
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1355
    moreover have "\<exists>\<^sub>F w in at z. fg w \<noteq> 0"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1356
      using fg_def fg_nconst by blast
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1357
    ultimately show ?thesis 
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1358
      using that zorder_exist[of fg z] fgn_def fgp_def by fastforce
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1359
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1360
  define r2 where "r2 = min fgr r1"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1361
  have "r2>0" using \<open>r1>0\<close> \<open>fgr>0\<close> unfolding r2_def by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1362
  show "fgn = fn + gn "
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1363
  proof (rule holomorphic_factor_unique)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1364
    show "\<forall>w \<in> ball z r2 - {z}. fg w = fgp w * (w - z) powi fgn \<and> fgp w \<noteq> 0 \<and> fg w = fp w * gp w * (w - z) powi (fn + gn) \<and> fp w * gp w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1365
      using fg_times fgp_nz fgr(2) r2_def by fastforce
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1366
  next
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1367
    show "fgp holomorphic_on ball z r2"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1368
      using fgr(1) r2_def by auto
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1369
  next
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1370
    show "(\<lambda>w. fp w * gp w) holomorphic_on ball z r2"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1371
      by (metis ball_subset_cball fr(1) gr(1) holomorphic_on_mult holomorphic_on_subset
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1372
          min.cobounded1 min.cobounded2 r1_def r2_def subset_ball)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1373
  qed (auto simp add: \<open>0 < r2\<close>)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1374
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1375
  have "fgp w = fp w *gp w" when w: "w \<in> ball z r2-{z}" for w
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1376
  proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1377
    have "w \<in> ball z r1 - {z}" "w \<in> cball z fgr - {z}" "w\<noteq>z" 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1378
      using w unfolding r2_def by auto
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1379
    then show ?thesis
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1380
      by (metis \<open>fgn = fn + gn\<close> eq_iff_diff_eq_0 fg_times fgr(2) power_int_eq_0_iff
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1381
          mult_right_cancel)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1382
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1383
  then show "\<forall>\<^sub>Fw in (at z). fgp w = fp w * gp w"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1384
    using \<open>r2>0\<close> unfolding eventually_at by (auto simp add: dist_commute)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1385
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1386
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1387
lemma
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1388
  fixes f g:: "complex \<Rightarrow> complex" and z::complex
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1389
  assumes f_iso: "isolated_singularity_at f z" and g_iso: "isolated_singularity_at g z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1390
      and f_ness: "not_essential f z" and g_ness: "not_essential g z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1391
      and fg_nconst: "\<exists>\<^sub>Fw in (at z). f w * g w\<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1392
  shows zorder_divide: "zorder (\<lambda>w. f w / g w) z = zorder f z - zorder g z" and
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1393
        zor_poly_divide: "\<forall>\<^sub>Fw in (at z). zor_poly (\<lambda>w. f w / g w) z w
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1394
                                       = zor_poly f z w  / zor_poly g z w"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1395
proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1396
  have f_nconst: "\<exists>\<^sub>Fw in (at z). f w \<noteq> 0" and g_nconst: "\<exists>\<^sub>Fw in (at z).g w\<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1397
    using fg_nconst by (auto elim!:frequently_elim1)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1398
  define vg where "vg=(\<lambda>w. inverse (g w))"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1399
  have 1: "isolated_singularity_at vg z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1400
    by (simp add: g_iso g_ness isolated_singularity_at_inverse vg_def)
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1401
  moreover have 2: "not_essential vg z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1402
    by (simp add: g_iso g_ness not_essential_inverse vg_def)
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1403
  moreover have 3: "\<exists>\<^sub>F w in at z. f w * vg w \<noteq> 0"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1404
    using fg_nconst vg_def by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1405
  ultimately have "zorder (\<lambda>w. f w * vg w) z = zorder f z + zorder vg z"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1406
    using zorder_times[OF f_iso _ f_ness] by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1407
  then show "zorder (\<lambda>w. f w / g w) z = zorder f z - zorder g z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1408
    using zorder_inverse[OF g_iso g_ness g_nconst,folded vg_def] unfolding vg_def
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1409
    by (auto simp add: field_simps)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1410
  have "\<forall>\<^sub>F w in at z. zor_poly (\<lambda>w. f w * vg w) z w = zor_poly f z w * zor_poly vg z w"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1411
    using zor_poly_times[OF f_iso _ f_ness,of vg] 1 2 3 by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1412
  then show "\<forall>\<^sub>Fw in (at z). zor_poly (\<lambda>w. f w / g w) z w = zor_poly f z w  / zor_poly g z w"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1413
    using zor_poly_inverse[OF g_iso g_ness g_nconst,folded vg_def] unfolding vg_def
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1414
    by eventually_elim (auto simp add: field_simps)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1415
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1416
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1417
lemma zorder_exist_zero:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1418
  fixes f:: "complex \<Rightarrow> complex" and z::complex
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1419
  defines "n \<equiv> zorder f z" and "g \<equiv> zor_poly f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1420
  assumes  holo: "f holomorphic_on S" and "open S" "connected S" "z\<in>S"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1421
      and non_const: "\<exists>w\<in>S. f w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1422
  shows "(if f z=0 then n > 0 else n=0) \<and> (\<exists>r. r>0 \<and> cball z r \<subseteq> S \<and> g holomorphic_on cball z r
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1423
    \<and> (\<forall>w\<in>cball z r. f w  = g w * (w-z) ^ nat n  \<and> g w \<noteq>0))"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1424
proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1425
  obtain r where "g z \<noteq> 0" and r: "r>0" "cball z r \<subseteq> S" "g holomorphic_on cball z r"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1426
            "(\<forall>w\<in>cball z r - {z}. f w = g w * (w-z) powi n \<and> g w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1427
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1428
    have "g z \<noteq> 0 \<and> (\<exists>r>0. g holomorphic_on cball z r
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1429
            \<and> (\<forall>w\<in>cball z r - {z}. f w = g w * (w-z) powi n \<and> g w \<noteq> 0))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1430
    proof (rule zorder_exist[of f z,folded g_def n_def])
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1431
      show "isolated_singularity_at f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1432
        using \<open>open S\<close> \<open>z\<in>S\<close> holo holomorphic_on_imp_analytic_at isolated_singularity_at_analytic 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1433
        by force 
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1434
      show "not_essential f z" unfolding not_essential_def
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1435
        using \<open>open S\<close> \<open>z\<in>S\<close> at_within_open continuous_on holo holomorphic_on_imp_continuous_on
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1436
        by fastforce
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1437
      have "\<forall>\<^sub>F w in at z. f w \<noteq> 0 \<and> w\<in>S"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1438
        using assms(4,5,6) holo non_const non_zero_neighbour_alt by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1439
      then show "\<exists>\<^sub>F w in at z. f w \<noteq> 0"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1440
        by (auto elim: eventually_frequentlyE)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1441
    qed
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1442
    then obtain r1 where "g z \<noteq> 0" "r1>0" and r1: "g holomorphic_on cball z r1"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1443
            "(\<forall>w\<in>cball z r1 - {z}. f w = g w * (w-z) powi n \<and> g w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1444
      by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1445
    obtain r2 where r2: "r2>0" "cball z r2 \<subseteq> S"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1446
      using assms(4,6) open_contains_cball_eq by blast
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1447
    define r3 where "r3 \<equiv> min r1 r2"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1448
    have "r3>0" "cball z r3 \<subseteq> S" using \<open>r1>0\<close> r2 unfolding r3_def by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1449
    moreover have "g holomorphic_on cball z r3"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1450
      using r1(1) unfolding r3_def by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1451
    moreover have "(\<forall>w\<in>cball z r3 - {z}. f w = g w * (w-z) powi n \<and> g w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1452
      using r1(2) unfolding r3_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1453
    ultimately show ?thesis using that[of r3] \<open>g z\<noteq>0\<close> by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1454
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1455
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1456
  have fz_lim: "f\<midarrow> z \<rightarrow> f z"
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1457
    by (metis assms(4,6) at_within_open continuous_on holo holomorphic_on_imp_continuous_on)
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1458
  have gz_lim: "g \<midarrow>z\<rightarrow>g z"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1459
    using r
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1460
    by (meson Elementary_Metric_Spaces.open_ball analytic_at analytic_at_imp_isCont 
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1461
        ball_subset_cball centre_in_ball holomorphic_on_subset isContD)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1462
  have if_0: "if f z=0 then n > 0 else n=0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1463
  proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1464
    have "(\<lambda>w. g w * (w-z) powi n) \<midarrow>z\<rightarrow> f z"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1465
      using fz_lim Lim_transform_within_open[where s="ball z r"] r by fastforce
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1466
    then have "(\<lambda>w. (g w * (w-z) powi n) / g w) \<midarrow>z\<rightarrow> f z/g z"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1467
      using gz_lim \<open>g z \<noteq> 0\<close> tendsto_divide by blast
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1468
    then have powi_tendsto: "(\<lambda>w. (w-z) powi n) \<midarrow>z\<rightarrow> f z/g z"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1469
      using Lim_transform_within_open[where s="ball z r"] r by fastforce
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1470
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1471
    have ?thesis when "n\<ge>0" "f z=0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1472
    proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1473
      have "(\<lambda>w. (w-z) ^ nat n) \<midarrow>z\<rightarrow> f z/g z"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1474
        using Lim_transform_within[OF powi_tendsto, where d=r]
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1475
        by (meson power_int_def r(1) that(1))
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1476
      then have *: "(\<lambda>w. (w-z) ^ nat n) \<midarrow>z\<rightarrow> 0" using \<open>f z=0\<close> by simp
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1477
      moreover have False when "n=0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1478
      proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1479
        have "(\<lambda>w. (w-z) ^ nat n) \<midarrow>z\<rightarrow> 1"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1480
          using \<open>n=0\<close> by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1481
        then show False using * using LIM_unique zero_neq_one by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1482
      qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1483
      ultimately show ?thesis using that by fastforce
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1484
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1485
    moreover have ?thesis when "n\<ge>0" "f z\<noteq>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1486
    proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1487
      have False when "n>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1488
      proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1489
        have "(\<lambda>w. (w-z) ^ nat n) \<midarrow>z\<rightarrow> f z/g z"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1490
          using Lim_transform_within[OF powi_tendsto, where d=r]
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1491
          by (meson \<open>0 \<le> n\<close> power_int_def r(1))
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1492
        moreover have "(\<lambda>w. (w-z) ^ nat n) \<midarrow>z\<rightarrow> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1493
          using \<open>n>0\<close> by (auto intro!:tendsto_eq_intros)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1494
        ultimately show False 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1495
          using \<open>f z\<noteq>0\<close> \<open>g z\<noteq>0\<close> LIM_unique divide_eq_0_iff by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1496
      qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1497
      then show ?thesis using that by force
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1498
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1499
    moreover have False when "n<0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1500
    proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1501
      have "(\<lambda>w. inverse ((w-z) ^ nat (- n))) \<midarrow>z\<rightarrow> f z/g z"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1502
        by (smt (verit) LIM_cong power_int_def power_inverse powi_tendsto that)
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1503
      moreover
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1504
      have "(\<lambda>w.((w-z) ^ nat (- n))) \<midarrow>z\<rightarrow> 0"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1505
        using that by (auto intro!:tendsto_eq_intros)
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1506
      ultimately
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1507
      have "(\<lambda>x. inverse ((x - z) ^ nat (- n)) * (x - z) ^ nat (- n)) \<midarrow>z\<rightarrow> 0" 
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1508
        using tendsto_mult by fastforce
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1509
      then have "(\<lambda>x. 1::complex) \<midarrow>z\<rightarrow> 0"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1510
        using Lim_transform_within_open by fastforce
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1511
      then show False 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1512
        using LIM_const_eq by fastforce
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1513
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1514
    ultimately show ?thesis by fastforce
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1515
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1516
  moreover have "f w  = g w * (w-z) ^ nat n  \<and> g w \<noteq>0" when "w\<in>cball z r" for w
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1517
  proof (cases "w=z")
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1518
    case True
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1519
    then have "f \<midarrow>z\<rightarrow>f w"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1520
      using fz_lim by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1521
    then have "(\<lambda>w. g w * (w-z) ^ nat n) \<midarrow>z\<rightarrow>f w"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1522
    proof (elim Lim_transform_within[OF _ \<open>r>0\<close>])
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1523
      fix x assume "0 < dist x z" "dist x z < r"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1524
      then have "x \<in> cball z r - {z}" "x\<noteq>z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1525
        unfolding cball_def by (auto simp add: dist_commute)
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1526
      then have "f x = g x * (x - z) powi n"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1527
        using r(4)[rule_format,of x] by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1528
      also have "... = g x * (x - z) ^ nat n"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1529
        by (smt (verit, best) if_0 int_nat_eq power_int_of_nat)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1530
      finally show "f x = g x * (x - z) ^ nat n" .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1531
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1532
    moreover have "(\<lambda>w. g w * (w-z) ^ nat n) \<midarrow>z\<rightarrow> g w * (w-z) ^ nat n"
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1533
      using True by (auto intro!:tendsto_eq_intros gz_lim)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1534
    ultimately have "f w = g w * (w-z) ^ nat n" using LIM_unique by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1535
    then show ?thesis using \<open>g z\<noteq>0\<close> True by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1536
  next
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1537
    case False
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1538
    then have "f w = g w * (w-z) powi n" "g w \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1539
      using r(4) that by auto
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1540
    then show ?thesis
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1541
      by (smt (verit, best) False if_0 int_nat_eq power_int_of_nat)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1542
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1543
  ultimately show ?thesis using r by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1544
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1545
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1546
lemma zorder_exist_pole:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1547
  fixes f:: "complex \<Rightarrow> complex" and z::complex
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1548
  defines "n\<equiv>zorder f z" and "g\<equiv>zor_poly f z"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1549
  assumes  holo: "f holomorphic_on S-{z}" and "open S" "z\<in>S" and "is_pole f z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1550
  shows "n < 0 \<and> g z\<noteq>0 \<and> (\<exists>r. r>0 \<and> cball z r \<subseteq> S \<and> g holomorphic_on cball z r
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1551
    \<and> (\<forall>w\<in>cball z r - {z}. f w  = g w / (w-z) ^ nat (- n) \<and> g w \<noteq>0))"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1552
proof -
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1553
  obtain r where "g z \<noteq> 0" and r: "r>0" "cball z r \<subseteq> S" "g holomorphic_on cball z r"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1554
            "(\<forall>w\<in>cball z r - {z}. f w = g w * (w-z) powi n \<and> g w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1555
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1556
    have "g z \<noteq> 0 \<and> (\<exists>r>0. g holomorphic_on cball z r
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1557
            \<and> (\<forall>w\<in>cball z r - {z}. f w = g w * (w-z) powi n \<and> g w \<noteq> 0))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1558
    proof (rule zorder_exist[of f z,folded g_def n_def])
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1559
      show "isolated_singularity_at f z" unfolding isolated_singularity_at_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1560
        using holo assms(4,5)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1561
        by (metis analytic_on_holomorphic centre_in_ball insert_Diff openE open_delete subset_insert_iff)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1562
      show "not_essential f z" unfolding not_essential_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1563
        using assms(4,6) at_within_open continuous_on holo holomorphic_on_imp_continuous_on
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1564
        by fastforce
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1565
      from non_zero_neighbour_pole[OF \<open>is_pole f z\<close>] show "\<exists>\<^sub>F w in at z. f w \<noteq> 0"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1566
        by (auto elim: eventually_frequentlyE)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1567
    qed
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1568
    then obtain r1 where "g z \<noteq> 0" "r1>0" and r1: "g holomorphic_on cball z r1"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1569
            "(\<forall>w\<in>cball z r1 - {z}. f w = g w * (w-z) powi n \<and> g w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1570
      by auto
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1571
    obtain r2 where r2: "r2>0" "cball z r2 \<subseteq> S"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1572
      using assms(4,5) open_contains_cball_eq by metis
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1573
    define r3 where "r3=min r1 r2"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1574
    have "r3>0" "cball z r3 \<subseteq> S" using \<open>r1>0\<close> r2 unfolding r3_def by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1575
    moreover have "g holomorphic_on cball z r3"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1576
      using r1(1) unfolding r3_def by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1577
    moreover have "(\<forall>w\<in>cball z r3 - {z}. f w = g w * (w-z) powi n \<and> g w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1578
      using r1(2) unfolding r3_def by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1579
    ultimately show ?thesis 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1580
      using that[of r3] \<open>g z\<noteq>0\<close> by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1581
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1582
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1583
  have "n<0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1584
  proof (rule ccontr)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1585
    assume " \<not> n < 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1586
    define c where "c=(if n=0 then g z else 0)"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1587
    have [simp]: "g \<midarrow>z\<rightarrow> g z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1588
      using r
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1589
      by (metis centre_in_ball continuous_on_interior holomorphic_on_imp_continuous_on
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1590
          interior_cball isContD)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1591
    have "\<forall>x \<in> ball z r. x \<noteq> z \<longrightarrow> f x = g x * (x - z) ^ nat n"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1592
      by (simp add: \<open>\<not> n < 0\<close> linorder_not_le power_int_def r)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1593
    then have "\<forall>\<^sub>F x in at z. f x = g x * (x - z) ^ nat n"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1594
      using centre_in_ball eventually_at_topological r(1) by blast
76897
a56e27f98763 continued proof simplification
paulson <lp15@cam.ac.uk>
parents: 76895
diff changeset
  1595
    moreover have "(\<lambda>x. g x * (x - z) ^ nat n) \<midarrow>z\<rightarrow> c"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1596
    proof (cases "n=0")
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1597
      case True
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1598
      then show ?thesis unfolding c_def by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1599
    next
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1600
      case False
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1601
      then have "(\<lambda>x. (x - z) ^ nat n) \<midarrow>z\<rightarrow> 0" using \<open>\<not> n < 0\<close>
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1602
        by (auto intro!:tendsto_eq_intros)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1603
      from tendsto_mult[OF _ this,of g "g z",simplified]
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1604
      show ?thesis unfolding c_def using False by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1605
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1606
    ultimately have "f \<midarrow>z\<rightarrow>c" using tendsto_cong by fast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1607
    then show False using \<open>is_pole f z\<close> at_neq_bot not_tendsto_and_filterlim_at_infinity
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1608
      unfolding is_pole_def by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1609
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1610
  moreover have "\<forall>w\<in>cball z r - {z}. f w  = g w / (w-z) ^ nat (- n) \<and> g w \<noteq>0"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1611
    using r(4) \<open>n<0\<close>
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1612
    by (smt (verit) inverse_eq_divide mult.right_neutral power_int_def power_inverse times_divide_eq_right)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1613
  ultimately show ?thesis 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1614
    using r \<open>g z\<noteq>0\<close> by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1615
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1616
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1617
lemma zorder_eqI:
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1618
  assumes "open S" "z \<in> S" "g holomorphic_on S" "g z \<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1619
  assumes fg_eq: "\<And>w. \<lbrakk>w \<in> S;w\<noteq>z\<rbrakk> \<Longrightarrow> f w = g w * (w-z) powi n"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1620
  shows   "zorder f z = n"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1621
proof -
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1622
  have "continuous_on S g" by (rule holomorphic_on_imp_continuous_on) fact
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1623
  moreover have "open (-{0::complex})" by auto
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1624
  ultimately have "open ((g -` (-{0})) \<inter> S)"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1625
    unfolding continuous_on_open_vimage[OF \<open>open S\<close>] by blast
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1626
  moreover from assms have "z \<in> (g -` (-{0})) \<inter> S" by auto
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1627
  ultimately obtain r where r: "r > 0" "cball z r \<subseteq>  S \<inter> (g -` (-{0}))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1628
    unfolding open_contains_cball by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1629
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1630
  let ?gg= "(\<lambda>w. g w * (w-z) powi n)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1631
  define P where "P = (\<lambda>n g r. 0 < r \<and> g holomorphic_on cball z r \<and> g z\<noteq>0
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1632
          \<and> (\<forall>w\<in>cball z r - {z}. f w = g w * (w-z) powi n \<and> g w\<noteq>0))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1633
  have "P n g r"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1634
    unfolding P_def using r assms(3,4,5) by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1635
  then have "\<exists>g r. P n g r" by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1636
  moreover have unique: "\<exists>!n. \<exists>g r. P n g r" unfolding P_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1637
  proof (rule holomorphic_factor_puncture)
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1638
    have "ball z r-{z} \<subseteq> S" using r using ball_subset_cball by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1639
    then have "?gg holomorphic_on ball z r-{z}"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1640
      using \<open>g holomorphic_on S\<close> r by (auto intro!: holomorphic_intros)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1641
    then have "f holomorphic_on ball z r - {z}"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1642
      by (smt (verit, best) DiffD2 \<open>ball z r-{z} \<subseteq> S\<close> fg_eq holomorphic_cong singleton_iff subset_iff)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1643
    then show "isolated_singularity_at f z" unfolding isolated_singularity_at_def
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1644
      using analytic_on_open open_delete r(1) by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1645
  next
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1646
    have "not_essential ?gg z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1647
    proof (intro singularity_intros)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1648
      show "not_essential g z"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1649
        by (meson \<open>continuous_on S g\<close> assms continuous_on_eq_continuous_at
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1650
            isCont_def not_essential_def)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1651
      show " \<forall>\<^sub>F w in at z. w - z \<noteq> 0" by (simp add: eventually_at_filter)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1652
      then show "LIM w at z. w - z :> at 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1653
        unfolding filterlim_at by (auto intro: tendsto_eq_intros)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1654
      show "isolated_singularity_at g z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1655
        by (meson Diff_subset open_ball analytic_on_holomorphic
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1656
            assms holomorphic_on_subset isolated_singularity_at_def openE)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1657
    qed
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1658
    moreover
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1659
    have "\<forall>\<^sub>F w in at z. g w * (w-z) powi n = f w"
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1660
      unfolding eventually_at_topological using assms fg_eq by force
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1661
    ultimately show "not_essential f z"
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1662
      using not_essential_transform by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1663
    show "\<exists>\<^sub>F w in at z. f w \<noteq> 0" unfolding frequently_at
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1664
    proof (intro strip)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1665
      fix d::real assume "0 < d"
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1666
      define z' where "z' \<equiv> z+min d r / 2"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1667
      have "z' \<noteq> z" " dist z' z < d "
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1668
        unfolding z'_def using \<open>d>0\<close> \<open>r>0\<close> by (auto simp add: dist_norm)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1669
      moreover have "f z' \<noteq> 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1670
      proof (subst fg_eq[OF _ \<open>z'\<noteq>z\<close>])
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  1671
        have "z' \<in> cball z r"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1672
          unfolding z'_def using \<open>r>0\<close> \<open>d>0\<close> by (auto simp add: dist_norm)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1673
        then show "z' \<in> S" using r(2) by blast
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1674
        show "g z' * (z' - z) powi n \<noteq> 0"
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1675
          using P_def \<open>P n g r\<close> \<open>z' \<in> cball z r\<close> \<open>z' \<noteq> z\<close> by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1676
      qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1677
      ultimately show "\<exists>x\<in>UNIV. x \<noteq> z \<and> dist x z < d \<and> f x \<noteq> 0" by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1678
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1679
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1680
  ultimately have "(THE n. \<exists>g r. P n g r) = n"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1681
    by (rule_tac the1_equality)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1682
  then show ?thesis unfolding zorder_def P_def by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1683
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1684
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1685
lemma simple_zeroI:
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1686
  assumes "open S" "z \<in> S" "g holomorphic_on S" "g z \<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1687
  assumes "\<And>w. w \<in> S \<Longrightarrow> f w = g w * (w-z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1688
  shows   "zorder f z = 1"
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1689
  using assms zorder_eqI by force
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1690
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1691
lemma higher_deriv_power:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1692
  shows   "(deriv ^^ j) (\<lambda>w. (w-z) ^ n) w =
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1693
             pochhammer (of_nat (Suc n - j)) j * (w-z) ^ (n - j)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1694
proof (induction j arbitrary: w)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1695
  case 0
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1696
  thus ?case by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1697
next
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1698
  case (Suc j w)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1699
  have "(deriv ^^ Suc j) (\<lambda>w. (w-z) ^ n) w = deriv ((deriv ^^ j) (\<lambda>w. (w-z) ^ n)) w"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1700
    by simp
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1701
  also have "(deriv ^^ j) (\<lambda>w. (w-z) ^ n) =
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1702
               (\<lambda>w. pochhammer (of_nat (Suc n - j)) j * (w-z) ^ (n - j))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1703
    using Suc by (intro Suc.IH ext)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1704
  also {
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1705
    have "(\<dots> has_field_derivative of_nat (n - j) *
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1706
               pochhammer (of_nat (Suc n - j)) j * (w-z) ^ (n - Suc j)) (at w)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1707
      using Suc.prems by (auto intro!: derivative_eq_intros)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1708
    also have "of_nat (n - j) * pochhammer (of_nat (Suc n - j)) j =
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1709
                 pochhammer (of_nat (Suc n - Suc j)) (Suc j)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1710
      by (cases "Suc j \<le> n", subst pochhammer_rec)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1711
         (use Suc.prems in \<open>simp_all add: algebra_simps Suc_diff_le pochhammer_0_left\<close>)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1712
    finally have "deriv (\<lambda>w. pochhammer (of_nat (Suc n - j)) j * (w-z) ^ (n - j)) w =
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1713
                    \<dots> * (w-z) ^ (n - Suc j)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1714
      by (rule DERIV_imp_deriv)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1715
  }
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1716
  finally show ?case .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1717
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1718
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1719
lemma zorder_zero_eqI:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1720
  assumes  f_holo: "f holomorphic_on S" and "open S" "z \<in> S"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1721
  assumes zero: "\<And>i. i < nat n \<Longrightarrow> (deriv ^^ i) f z = 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1722
  assumes nz: "(deriv ^^ nat n) f z \<noteq> 0" and "n\<ge>0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1723
  shows   "zorder f z = n"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1724
proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1725
  obtain r where [simp]: "r>0" and "ball z r \<subseteq> S"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1726
    using \<open>open S\<close> \<open>z\<in>S\<close> openE by blast
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1727
  have nz': "\<exists>w\<in>ball z r. f w \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1728
  proof (rule ccontr)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1729
    assume "\<not> (\<exists>w\<in>ball z r. f w \<noteq> 0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1730
    then have "eventually (\<lambda>u. f u = 0) (nhds z)"
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1731
      using open_ball \<open>0 < r\<close> centre_in_ball eventually_nhds by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1732
    then have "(deriv ^^ nat n) f z = (deriv ^^ nat n) (\<lambda>_. 0) z"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1733
      by (intro higher_deriv_cong_ev) auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1734
    also have "(deriv ^^ nat n) (\<lambda>_. 0) z = 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1735
      by (induction n) simp_all
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1736
    finally show False using nz by contradiction
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1737
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1738
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1739
  define zn g where "zn = zorder f z" and "g = zor_poly f z"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1740
  obtain e where e_if: "if f z = 0 then 0 < zn else zn = 0" and
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1741
            [simp]: "e>0" and "cball z e \<subseteq> ball z r" and
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1742
            g_holo: "g holomorphic_on cball z e" and
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1743
            e_fac: "(\<forall>w\<in>cball z e. f w = g w * (w-z) ^ nat zn \<and> g w \<noteq> 0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1744
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1745
    have "f holomorphic_on ball z r"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1746
      using f_holo \<open>ball z r \<subseteq> S\<close> by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1747
    from that zorder_exist_zero[of f "ball z r" z,simplified,OF this nz',folded zn_def g_def]
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1748
    show thesis by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1749
  qed
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1750
  then obtain "zn \<ge> 0" "g z \<noteq> 0"
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1751
    by (metis centre_in_cball less_le_not_le order_refl)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1752
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1753
  define A where "A \<equiv> (\<lambda>i. of_nat (i choose (nat zn)) * fact (nat zn) * (deriv ^^ (i - nat zn)) g z)"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1754
  have deriv_A: "(deriv ^^ i) f z = (if zn \<le> int i then A i else 0)" for i
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1755
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1756
    have "eventually (\<lambda>w. w \<in> ball z e) (nhds z)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1757
      using \<open>cball z e \<subseteq> ball z r\<close> \<open>e>0\<close> by (intro eventually_nhds_in_open) auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1758
    hence "eventually (\<lambda>w. f w = (w-z) ^ (nat zn) * g w) (nhds z)"
76900
830597d13d6d final tidying of theorems
paulson <lp15@cam.ac.uk>
parents: 76897
diff changeset
  1759
      using e_fac eventually_mono by fastforce
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1760
    hence "(deriv ^^ i) f z = (deriv ^^ i) (\<lambda>w. (w-z) ^ nat zn * g w) z"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1761
      by (intro higher_deriv_cong_ev) auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1762
    also have "\<dots> = (\<Sum>j=0..i. of_nat (i choose j) *
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1763
                       (deriv ^^ j) (\<lambda>w. (w-z) ^ nat zn) z * (deriv ^^ (i - j)) g z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1764
      using g_holo \<open>e>0\<close>
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1765
      by (intro higher_deriv_mult[of _ "ball z e"]) (auto intro!: holomorphic_intros)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1766
    also have "\<dots> = (\<Sum>j=0..i. if j = nat zn then
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1767
                    of_nat (i choose nat zn) * fact (nat zn) * (deriv ^^ (i - nat zn)) g z else 0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1768
    proof (intro sum.cong refl, goal_cases)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1769
      case (1 j)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1770
      have "(deriv ^^ j) (\<lambda>w. (w-z) ^ nat zn) z =
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1771
              pochhammer (of_nat (Suc (nat zn) - j)) j * 0 ^ (nat zn - j)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1772
        by (subst higher_deriv_power) auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1773
      also have "\<dots> = (if j = nat zn then fact j else 0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1774
        by (auto simp: not_less pochhammer_0_left pochhammer_fact)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1775
      also have "of_nat (i choose j) * \<dots> * (deriv ^^ (i - j)) g z =
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1776
                   (if j = nat zn then of_nat (i choose (nat zn)) * fact (nat zn)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1777
                        * (deriv ^^ (i - nat zn)) g z else 0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1778
        by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1779
      finally show ?case .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1780
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1781
    also have "\<dots> = (if i \<ge> zn then A i else 0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1782
      by (auto simp: A_def)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1783
    finally show "(deriv ^^ i) f z = \<dots>" .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1784
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1785
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1786
  have False when "n<zn"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1787
    using deriv_A[of "nat n"] that \<open>n\<ge>0\<close> by (simp add: nz) 
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1788
  moreover have "n\<le>zn"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1789
  proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1790
    have "g z \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1791
      by (simp add: \<open>g z \<noteq> 0\<close>)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1792
    then have "(deriv ^^ nat zn) f z \<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1793
      using deriv_A[of "nat zn"] by(auto simp add: A_def)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1794
    then have "nat zn \<ge> nat n" using zero[of "nat zn"] by linarith
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1795
    moreover have "zn\<ge>0" using e_if by (auto split: if_splits)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1796
    ultimately show ?thesis using nat_le_eq_zle by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1797
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1798
  ultimately show ?thesis unfolding zn_def by fastforce
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1799
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1800
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1801
lemma
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1802
  assumes "eventually (\<lambda>z. f z = g z) (at z)" "z = z'"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1803
  shows zorder_cong: "zorder f z = zorder g z'" and zor_poly_cong: "zor_poly f z = zor_poly g z'"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1804
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1805
  define P where "P = (\<lambda>ff n h r. 0 < r \<and> h holomorphic_on cball z r \<and> h z\<noteq>0
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1806
                    \<and> (\<forall>w\<in>cball z r - {z}. ff w = h w * (w-z) powi n \<and> h w\<noteq>0))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1807
  have "(\<exists>r. P f n h r) = (\<exists>r. P g n h r)" for n h
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1808
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1809
    have *: "\<exists>r. P g n h r" if "\<exists>r. P f n h r" and "eventually (\<lambda>x. f x = g x) (at z)" for f g
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1810
    proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1811
      from that(1) obtain r1 where r1_P: "P f n h r1" by auto
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1812
      from that(2) obtain r2 where "r2>0" and r2_dist: "\<forall>x. x \<noteq> z \<and> dist x z \<le> r2 \<longrightarrow> f x = g x"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1813
        unfolding eventually_at_le by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1814
      define r where "r=min r1 r2"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1815
      have "r>0" "h z\<noteq>0" using r1_P \<open>r2>0\<close> unfolding r_def P_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1816
      moreover have "h holomorphic_on cball z r"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1817
        using r1_P unfolding P_def r_def by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1818
      moreover have "g w = h w * (w-z) powi n \<and> h w \<noteq> 0" when "w\<in>cball z r - {z}" for w
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1819
      proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1820
        have "f w = h w * (w-z) powi n \<and> h w \<noteq> 0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1821
          using r1_P that unfolding P_def r_def by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1822
        moreover have "f w=g w"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1823
          using r2_dist that by (simp add: dist_commute r_def)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1824
        ultimately show ?thesis by simp
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1825
      qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1826
      ultimately show ?thesis unfolding P_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1827
    qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1828
    from assms have eq': "eventually (\<lambda>z. g z = f z) (at z)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1829
      by (simp add: eq_commute)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1830
    show ?thesis
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1831
      using "*" assms(1) eq' by blast
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1832
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1833
  then show "zorder f z = zorder g z'" "zor_poly f z = zor_poly g z'"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1834
      using \<open>z=z'\<close> unfolding P_def zorder_def zor_poly_def by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1835
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1836
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1837
lemma zorder_times_analytic':
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1838
  assumes "isolated_singularity_at f z" "not_essential f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1839
  assumes "g analytic_on {z}" "frequently (\<lambda>z. f z * g z \<noteq> 0) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1840
  shows   "zorder (\<lambda>x. f x * g x) z = zorder f z + zorder g z"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1841
  using assms isolated_singularity_at_analytic not_essential_analytic zorder_times by blast
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1842
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1843
lemma zorder_cmult:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1844
  assumes "c \<noteq> 0"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1845
  shows   "zorder (\<lambda>z. c * f z) z = zorder f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1846
proof -
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1847
  define P where
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1848
    "P = (\<lambda>f n h r. 0 < r \<and> h holomorphic_on cball z r \<and>
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1849
                    h z \<noteq> 0 \<and> (\<forall>w\<in>cball z r - {z}. f w = h w * (w-z) powi n \<and> h w \<noteq> 0))"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1850
  have *: "P (\<lambda>x. c * f x) n (\<lambda>x. c * h x) r" 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1851
    if "P f n h r" "c \<noteq> 0" for f n h r c
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1852
    using that unfolding P_def by (auto intro!: holomorphic_intros)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1853
  have "(\<exists>h r. P (\<lambda>x. c * f x) n h r) \<longleftrightarrow> (\<exists>h r. P f n h r)" for n
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1854
    using *[of f n _ _ c] *[of "\<lambda>x. c * f x" n _ _ "inverse c"] \<open>c \<noteq> 0\<close>
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1855
    by (fastforce simp: field_simps)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1856
  hence "(THE n. \<exists>h r. P (\<lambda>x. c * f x) n h r) = (THE n. \<exists>h r. P f n h r)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1857
    by simp
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1858
  thus ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1859
    by (simp add: zorder_def P_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1860
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  1861
79945
ca004ccf2352 New material from a variety of sources (including AFP)
paulson <lp15@cam.ac.uk>
parents: 78517
diff changeset
  1862
lemma zorder_uminus [simp]: "zorder (\<lambda>z. -f z) z = zorder f z"
ca004ccf2352 New material from a variety of sources (including AFP)
paulson <lp15@cam.ac.uk>
parents: 78517
diff changeset
  1863
  using zorder_cmult[of "-1" f] by simp
ca004ccf2352 New material from a variety of sources (including AFP)
paulson <lp15@cam.ac.uk>
parents: 78517
diff changeset
  1864
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1865
lemma zorder_nonzero_div_power:
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1866
  assumes sz: "open S" "z \<in> S" "f holomorphic_on S" "f z \<noteq> 0" and "n > 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1867
  shows  "zorder (\<lambda>w. f w / (w-z) ^ n) z = - n"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1868
  by (intro zorder_eqI [OF sz]) (simp add: inverse_eq_divide power_int_minus)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1869
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1870
lemma zor_poly_eq:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1871
  assumes "isolated_singularity_at f z" "not_essential f z" "\<exists>\<^sub>F w in at z. f w \<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1872
  shows "eventually (\<lambda>w. zor_poly f z w = f w * (w-z) powi - zorder f z) (at z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1873
proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1874
  obtain r where r: "r>0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1875
       "(\<forall>w\<in>cball z r - {z}. f w = zor_poly f z w * (w-z) powi (zorder f z))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1876
    using zorder_exist[OF assms] by blast
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1877
  then have *: "\<forall>w\<in>ball z r - {z}. zor_poly f z w = f w * (w-z) powi - zorder f z"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1878
    by (auto simp: field_simps power_int_minus)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1879
  have "eventually (\<lambda>w. w \<in> ball z r - {z}) (at z)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1880
    using r eventually_at_ball'[of r z UNIV] by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1881
  thus ?thesis by eventually_elim (insert *, auto)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1882
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1883
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1884
lemma zor_poly_zero_eq:
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  1885
  assumes "f holomorphic_on S" "open S" "connected S" "z \<in> S" "\<exists>w\<in>S. f w \<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1886
  shows "eventually (\<lambda>w. zor_poly f z w = f w / (w-z) ^ nat (zorder f z)) (at z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1887
proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1888
  obtain r where r: "r>0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1889
       "(\<forall>w\<in>cball z r - {z}. f w = zor_poly f z w * (w-z) ^ nat (zorder f z))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1890
    using zorder_exist_zero[OF assms] by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1891
  then have *: "\<forall>w\<in>ball z r - {z}. zor_poly f z w = f w / (w-z) ^ nat (zorder f z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1892
    by (auto simp: field_simps powr_minus)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1893
  have "eventually (\<lambda>w. w \<in> ball z r - {z}) (at z)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1894
    using r eventually_at_ball'[of r z UNIV] by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1895
  thus ?thesis by eventually_elim (insert *, auto)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1896
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1897
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1898
lemma zor_poly_pole_eq:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1899
  assumes f_iso: "isolated_singularity_at f z" "is_pole f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1900
  shows "eventually (\<lambda>w. zor_poly f z w = f w * (w-z) ^ nat (- zorder f z)) (at z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1901
proof -
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1902
  obtain e where [simp]: "e>0" and f_holo: "f holomorphic_on ball z e - {z}"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1903
    using f_iso analytic_imp_holomorphic unfolding isolated_singularity_at_def by blast
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1904
  obtain r where r: "r>0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1905
       "(\<forall>w\<in>cball z r - {z}. f w = zor_poly f z w / (w-z) ^ nat (- zorder f z))"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1906
    using zorder_exist_pole[OF f_holo,simplified,OF \<open>is_pole f z\<close>] by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1907
  then have *: "\<forall>w\<in>ball z r - {z}. zor_poly f z w = f w * (w-z) ^ nat (- zorder f z)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1908
    by (auto simp: field_simps)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1909
  have "eventually (\<lambda>w. w \<in> ball z r - {z}) (at z)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1910
    using r eventually_at_ball'[of r z UNIV] by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1911
  thus ?thesis by eventually_elim (insert *, auto)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1912
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1913
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1914
lemma zor_poly_eqI:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1915
  fixes f :: "complex \<Rightarrow> complex" and z0 :: complex
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1916
  defines "n \<equiv> zorder f z0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1917
  assumes "isolated_singularity_at f z0" "not_essential f z0" "\<exists>\<^sub>F w in at z0. f w \<noteq> 0"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1918
  assumes lim: "((\<lambda>x. f (g x) * (g x - z0) powi - n) \<longlongrightarrow> c) F"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1919
  assumes g: "filterlim g (at z0) F" and "F \<noteq> bot"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1920
  shows   "zor_poly f z0 z0 = c"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1921
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1922
  from zorder_exist[OF assms(2-4)] obtain r where
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1923
    r: "r > 0" "zor_poly f z0 holomorphic_on cball z0 r"
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1924
       "\<And>w. w \<in> cball z0 r - {z0} \<Longrightarrow> f w = zor_poly f z0 w * (w - z0) powi n"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1925
    unfolding n_def by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1926
  from r(1) have "eventually (\<lambda>w. w \<in> ball z0 r \<and> w \<noteq> z0) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1927
    using eventually_at_ball'[of r z0 UNIV] by auto
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1928
  hence "eventually (\<lambda>w. zor_poly f z0 w = f w * (w - z0) powi - n) (at z0)"
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1929
    by eventually_elim (insert r, auto simp: field_simps power_int_minus)
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1930
  moreover have "continuous_on (ball z0 r) (zor_poly f z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1931
    using r by (intro holomorphic_on_imp_continuous_on) auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1932
  with r have "isCont (zor_poly f z0) z0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1933
    by (auto simp: continuous_on_eq_continuous_at)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1934
  hence "(zor_poly f z0 \<longlongrightarrow> zor_poly f z0 z0) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1935
    unfolding isCont_def .
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1936
  ultimately have "((\<lambda>w. f w * (w - z0) powi - n) \<longlongrightarrow> zor_poly f z0 z0) (at z0)"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1937
    by (blast intro: Lim_transform_eventually)
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  1938
  hence "((\<lambda>x. f (g x) * (g x - z0) powi - n) \<longlongrightarrow> zor_poly f z0 z0) F"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1939
    by (rule filterlim_compose[OF _ g])
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1940
  from tendsto_unique[OF \<open>F \<noteq> bot\<close> this lim] show ?thesis .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1941
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1942
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1943
lemma zor_poly_zero_eqI:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1944
  fixes f :: "complex \<Rightarrow> complex" and z0 :: complex
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1945
  defines "n \<equiv> zorder f z0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1946
  assumes "f holomorphic_on A" "open A" "connected A" "z0 \<in> A" "\<exists>z\<in>A. f z \<noteq> 0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1947
  assumes lim: "((\<lambda>x. f (g x) / (g x - z0) ^ nat n) \<longlongrightarrow> c) F"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1948
  assumes g: "filterlim g (at z0) F" and "F \<noteq> bot"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1949
  shows   "zor_poly f z0 z0 = c"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1950
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1951
  from zorder_exist_zero[OF assms(2-6)] obtain r where
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1952
    r: "r > 0" "cball z0 r \<subseteq> A" "zor_poly f z0 holomorphic_on cball z0 r"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1953
       "\<And>w. w \<in> cball z0 r \<Longrightarrow> f w = zor_poly f z0 w * (w - z0) ^ nat n"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1954
    unfolding n_def by blast
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1955
  from r(1) have "eventually (\<lambda>w. w \<in> ball z0 r \<and> w \<noteq> z0) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1956
    using eventually_at_ball'[of r z0 UNIV] by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1957
  hence "eventually (\<lambda>w. zor_poly f z0 w = f w / (w - z0) ^ nat n) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1958
    by eventually_elim (insert r, auto simp: field_simps)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1959
  moreover have "continuous_on (ball z0 r) (zor_poly f z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1960
    using r by (intro holomorphic_on_imp_continuous_on) auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1961
  with r(1,2) have "isCont (zor_poly f z0) z0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1962
    by (auto simp: continuous_on_eq_continuous_at)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1963
  hence "(zor_poly f z0 \<longlongrightarrow> zor_poly f z0 z0) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1964
    unfolding isCont_def .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1965
  ultimately have "((\<lambda>w. f w / (w - z0) ^ nat n) \<longlongrightarrow> zor_poly f z0 z0) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1966
    by (blast intro: Lim_transform_eventually)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1967
  hence "((\<lambda>x. f (g x) / (g x - z0) ^ nat n) \<longlongrightarrow> zor_poly f z0 z0) F"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1968
    by (rule filterlim_compose[OF _ g])
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1969
  from tendsto_unique[OF \<open>F \<noteq> bot\<close> this lim] show ?thesis .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1970
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1971
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1972
lemma zor_poly_pole_eqI:
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1973
  fixes f :: "complex \<Rightarrow> complex" and z0 :: complex
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1974
  defines "n \<equiv> zorder f z0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1975
  assumes f_iso: "isolated_singularity_at f z0" and "is_pole f z0"
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1976
  assumes lim: "((\<lambda>x. f (g x) * (g x - z0) ^ nat (-n)) \<longlongrightarrow> c) F"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1977
  assumes g: "filterlim g (at z0) F" and "F \<noteq> bot"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1978
  shows   "zor_poly f z0 z0 = c"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1979
proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1980
  obtain r where r: "r > 0"  "zor_poly f z0 holomorphic_on cball z0 r"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1981
  proof -
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1982
    have "\<exists>\<^sub>F w in at z0. f w \<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1983
      using non_zero_neighbour_pole[OF \<open>is_pole f z0\<close>] 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1984
      by (auto elim: eventually_frequentlyE)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1985
    moreover have "not_essential f z0" 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1986
      unfolding not_essential_def using \<open>is_pole f z0\<close> by simp
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1987
    ultimately show ?thesis 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  1988
      using that zorder_exist[OF f_iso,folded n_def] by auto
71201
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1989
  qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1990
  from r(1) have "eventually (\<lambda>w. w \<in> ball z0 r \<and> w \<noteq> z0) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1991
    using eventually_at_ball'[of r z0 UNIV] by auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1992
  have "eventually (\<lambda>w. zor_poly f z0 w = f w * (w - z0) ^ nat (-n)) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1993
    using zor_poly_pole_eq[OF f_iso \<open>is_pole f z0\<close>] unfolding n_def .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1994
  moreover have "continuous_on (ball z0 r) (zor_poly f z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1995
    using r by (intro holomorphic_on_imp_continuous_on) auto
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1996
  with r(1,2) have "isCont (zor_poly f z0) z0"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1997
    by (auto simp: continuous_on_eq_continuous_at)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1998
  hence "(zor_poly f z0 \<longlongrightarrow> zor_poly f z0 z0) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  1999
    unfolding isCont_def .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  2000
  ultimately have "((\<lambda>w. f w * (w - z0) ^ nat (-n)) \<longlongrightarrow> zor_poly f z0 z0) (at z0)"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  2001
    by (blast intro: Lim_transform_eventually)
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  2002
  hence "((\<lambda>x. f (g x) * (g x - z0) ^ nat (-n)) \<longlongrightarrow> zor_poly f z0 z0) F"
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  2003
    by (rule filterlim_compose[OF _ g])
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  2004
  from tendsto_unique[OF \<open>F \<noteq> bot\<close> this lim] show ?thesis .
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  2005
qed
6617fb368a06 Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff changeset
  2006
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2007
lemma
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2008
  assumes "is_pole f (x :: complex)" "open A" "x \<in> A"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2009
  assumes "\<And>y. y \<in> A - {x} \<Longrightarrow> (f has_field_derivative f' y) (at y)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2010
  shows   is_pole_deriv': "is_pole f' x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2011
    and   zorder_deriv':  "zorder f' x = zorder f x - 1"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2012
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2013
  have holo: "f holomorphic_on A - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2014
    using assms by (subst holomorphic_on_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2015
  obtain r where r: "r > 0" "ball x r \<subseteq> A"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2016
    using assms(2,3) openE by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2017
  moreover have "open (ball x r - {x})"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2018
    by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2019
  ultimately have "isolated_singularity_at f x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2020
    by (auto simp: isolated_singularity_at_def analytic_on_open
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2021
             intro!: exI[of _ r] holomorphic_on_subset[OF holo])
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2022
  hence ev: "\<forall>\<^sub>F w in at x. zor_poly f x w = f w * (w-x) ^ nat (- zorder f x)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2023
    using \<open>is_pole f x\<close> zor_poly_pole_eq by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2024
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2025
  define P where "P = zor_poly f x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2026
  define n where "n = nat (-zorder f x)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2027
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2028
  obtain r where r: "r > 0" "cball x r \<subseteq> A" "P holomorphic_on cball x r" "zorder f x < 0" "P x \<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2029
    "\<forall>w\<in>cball x r - {x}. f w = P w / (w-x) ^ n \<and> P w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2030
    using P_def assms holo n_def zorder_exist_pole by blast
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2031
  have n: "n > 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2032
    using r(4) by (auto simp: n_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2033
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2034
  have [derivative_intros]: "(P has_field_derivative deriv P w) (at w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2035
    if "w \<in> ball x r" for w
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2036
    using that by (intro holomorphic_derivI[OF holomorphic_on_subset[OF r(3), of "ball x r"]]) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2037
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2038
  define D where "D = (\<lambda>w. (deriv P w * (w-x) - of_nat n * P w) / (w-x) ^ (n + 1))"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2039
  define n' where "n' = n - 1"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2040
  have n': "n = Suc n'"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2041
    using n by (simp add: n'_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2042
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2043
  have "eventually (\<lambda>w. w \<in> ball x r) (nhds x)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2044
    using \<open>r > 0\<close> by (intro eventually_nhds_in_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2045
  hence ev'': "eventually (\<lambda>w. w \<in> ball x r - {x}) (at x)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2046
    by (auto simp: eventually_at_filter elim: eventually_mono)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2047
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2048
  {
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2049
    fix w assume w: "w \<in> ball x r - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2050
    have ev': "eventually (\<lambda>w. w \<in> ball x r - {x}) (nhds w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2051
      using w by (intro eventually_nhds_in_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2052
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2053
    have \<section>: "(deriv P w * (w-x) ^ n - P w * (n * (w-x) ^ (n-1))) / ((w-x) ^ n * (w-x) ^ n) = D w"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2054
      using w n' by (simp add: divide_simps D_def) (simp add: algebra_simps)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2055
    have "((\<lambda>w. P w / (w-x) ^ n) has_field_derivative D w) (at w)"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2056
      by (rule derivative_eq_intros refl | use w \<section> in force)+
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2057
    also have "?this \<longleftrightarrow> (f has_field_derivative D w) (at w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2058
      using r by (intro has_field_derivative_cong_ev refl eventually_mono[OF ev']) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2059
    finally have "(f has_field_derivative D w) (at w)" .
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2060
    moreover have "(f has_field_derivative f' w) (at w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2061
      using w r by (intro assms) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2062
    ultimately have "D w = f' w"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2063
      using DERIV_unique by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2064
  } note D_eq = this
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2065
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2066
  have "is_pole D x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2067
    unfolding D_def using n \<open>r > 0\<close> \<open>P x \<noteq> 0\<close>
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2068
    by (intro is_pole_basic[where A = "ball x r"] holomorphic_intros holomorphic_on_subset[OF r(3)]) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2069
  also have "?this \<longleftrightarrow> is_pole f' x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2070
    by (intro is_pole_cong eventually_mono[OF ev''] D_eq) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2071
  finally show "is_pole f' x" .
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2072
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2073
  have "zorder f' x = -int (Suc n)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2074
  proof (rule zorder_eqI)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2075
    show "open (ball x r)" "x \<in> ball x r"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2076
      using \<open>r > 0\<close> by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2077
    show "f' w = (deriv P w * (w-x) - of_nat n * P w) * (w-x) powi (- int (Suc n))"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2078
      if "w \<in> ball x r" "w \<noteq> x" for w
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  2079
      using that D_eq[of w] n by (auto simp: D_def power_int_diff power_int_minus powr_nat' divide_simps)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2080
  qed (use r n in \<open>auto intro!: holomorphic_intros\<close>)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2081
  thus "zorder f' x = zorder f x - 1"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2082
    using n by (simp add: n_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2083
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2084
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2085
lemma
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2086
  assumes "is_pole f (x :: complex)" "isolated_singularity_at f x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2087
  shows   is_pole_deriv: "is_pole (deriv f) x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2088
    and   zorder_deriv:  "zorder (deriv f) x = zorder f x - 1"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2089
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2090
  from assms(2) obtain r where r: "r > 0" "f analytic_on ball x r - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2091
    by (auto simp: isolated_singularity_at_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2092
  hence holo: "f holomorphic_on ball x r - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2093
    by (subst (asm) analytic_on_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2094
  have *: "x \<in> ball x r" "open (ball x r)" "open (ball x r - {x})"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2095
    using \<open>r > 0\<close> by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2096
  show "is_pole (deriv f) x" "zorder (deriv f) x = zorder f x - 1"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2097
    by (meson "*" assms(1) holo holomorphic_derivI is_pole_deriv' zorder_deriv')+
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2098
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2099
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2100
lemma removable_singularity_deriv':
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2101
  assumes "f \<midarrow>x\<rightarrow> c" "x \<in> A" "open (A :: complex set)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2102
  assumes "\<And>y. y \<in> A - {x} \<Longrightarrow> (f has_field_derivative f' y) (at y)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2103
  shows   "\<exists>c. f' \<midarrow>x\<rightarrow> c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2104
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2105
  have holo: "f holomorphic_on A - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2106
    using assms by (subst holomorphic_on_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2107
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2108
  define g where "g = (\<lambda>y. if y = x then c else f y)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2109
  have deriv_g_eq: "deriv g y = f' y" if "y \<in> A - {x}" for y
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2110
  proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2111
    have ev: "eventually (\<lambda>y. y \<in> A - {x}) (nhds y)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2112
      using that assms by (intro eventually_nhds_in_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2113
    have "(f has_field_derivative f' y) (at y)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2114
      using assms that by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2115
    also have "?this \<longleftrightarrow> (g has_field_derivative f' y) (at y)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2116
      by (intro has_field_derivative_cong_ev refl eventually_mono[OF ev]) (auto simp: g_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2117
    finally show ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2118
      by (intro DERIV_imp_deriv assms)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2119
  qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2120
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2121
  have "g holomorphic_on A"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2122
    unfolding g_def using assms assms(1) holo 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2123
    by (intro removable_singularity) auto
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2124
  hence "deriv g holomorphic_on A"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2125
    by (intro holomorphic_deriv assms)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2126
  hence "continuous_on A (deriv g)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2127
    by (meson holomorphic_on_imp_continuous_on)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2128
  hence "(deriv g \<longlongrightarrow> deriv g x) (at x within A)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2129
    using assms by (auto simp: continuous_on_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2130
  also have "?this \<longleftrightarrow> (f' \<longlongrightarrow> deriv g x) (at x within A)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2131
    by (intro filterlim_cong refl) (auto simp: eventually_at_filter deriv_g_eq)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2132
  finally have "f' \<midarrow>x\<rightarrow> deriv g x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2133
    using \<open>open A\<close> \<open>x \<in> A\<close> by (meson tendsto_within_open)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2134
  thus ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2135
    by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2136
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2137
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2138
lemma removable_singularity_deriv:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2139
  assumes "f \<midarrow>x\<rightarrow> c" "isolated_singularity_at f x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2140
  shows   "\<exists>c. deriv f \<midarrow>x\<rightarrow> c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2141
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2142
  from assms(2) obtain r where r: "r > 0" "f analytic_on ball x r - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2143
    by (auto simp: isolated_singularity_at_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2144
  hence holo: "f holomorphic_on ball x r - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2145
    using analytic_imp_holomorphic by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2146
  show ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2147
    using assms(1)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2148
  proof (rule removable_singularity_deriv')
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2149
    show "x \<in> ball x r" "open (ball x r)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2150
      using \<open>r > 0\<close> by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2151
  qed (auto intro!: holomorphic_derivI[OF holo])
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2152
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2153
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2154
lemma not_essential_deriv':
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2155
  assumes "not_essential f x" "x \<in> A" "open A"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2156
  assumes "\<And>y. y \<in> A - {x} \<Longrightarrow> (f has_field_derivative f' y) (at y)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2157
  shows   "not_essential f' x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2158
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2159
  have holo: "f holomorphic_on A - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2160
    using assms by (subst holomorphic_on_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2161
  from assms consider "is_pole f x" | c where "f \<midarrow>x\<rightarrow> c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2162
    by (auto simp: not_essential_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2163
  thus ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2164
  proof cases
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2165
    case 1
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2166
    thus ?thesis
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2167
      using assms is_pole_deriv' by blast
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2168
  next
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2169
    case (2 c)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2170
    thus ?thesis
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2171
      by (meson assms removable_singularity_deriv' tendsto_imp_not_essential)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2172
  qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2173
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2174
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2175
lemma not_essential_deriv[singularity_intros]:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2176
  assumes "not_essential f x" "isolated_singularity_at f x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2177
  shows   "not_essential (deriv f) x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2178
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2179
  from assms(2) obtain r where r: "r > 0" "f analytic_on ball x r - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2180
    by (auto simp: isolated_singularity_at_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2181
  hence holo: "f holomorphic_on ball x r - {x}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2182
    by (subst (asm) analytic_on_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2183
  show ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2184
    using assms(1)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2185
  proof (rule not_essential_deriv')
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2186
    show "x \<in> ball x r" "open (ball x r)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2187
      using \<open>r > 0\<close> by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2188
  qed (auto intro!: holomorphic_derivI[OF holo])
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2189
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2190
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2191
lemma not_essential_frequently_0_imp_tendsto_0:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2192
  fixes f :: "complex \<Rightarrow> complex"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2193
  assumes sing: "isolated_singularity_at f z" "not_essential f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2194
  assumes freq: "frequently (\<lambda>z. f z = 0) (at z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2195
  shows   "f \<midarrow>z\<rightarrow> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2196
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2197
  from freq obtain g :: "nat \<Rightarrow> complex" where g: "filterlim g (at z) at_top" "\<And>n. f (g n) = 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2198
    using frequently_atE by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2199
  have "eventually (\<lambda>x. f (g x) = 0) sequentially"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2200
    using g by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2201
  hence fg: "(\<lambda>x. f (g x)) \<longlonglongrightarrow> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2202
    by (simp add: tendsto_eventually)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2203
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2204
  from assms(2) consider c where "f \<midarrow>z\<rightarrow> c" | "is_pole f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2205
    unfolding not_essential_def by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2206
  thus ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2207
  proof cases
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2208
    case (1 c)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2209
    have "(\<lambda>x. f (g x)) \<longlonglongrightarrow> c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2210
      by (rule filterlim_compose[OF 1 g(1)])
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2211
    with fg have "c = 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2212
      using LIMSEQ_unique by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2213
    with 1 show ?thesis by simp
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2214
  next
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2215
    case 2
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2216
    have "filterlim (\<lambda>x. f (g x)) at_infinity sequentially"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2217
      using "2" filterlim_compose g(1) is_pole_def by blast
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2218
    with fg have False
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2219
      by (meson not_tendsto_and_filterlim_at_infinity sequentially_bot)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2220
    thus ?thesis ..
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2221
  qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2222
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2224
lemma not_essential_frequently_0_imp_eventually_0:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2225
  fixes f :: "complex \<Rightarrow> complex"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2226
  assumes sing: "isolated_singularity_at f z" "not_essential f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2227
  assumes freq: "frequently (\<lambda>z. f z = 0) (at z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2228
  shows   "eventually (\<lambda>z. f z = 0) (at z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2229
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2230
  from sing obtain r where r: "r > 0" and "f analytic_on ball z r - {z}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2231
    by (auto simp: isolated_singularity_at_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2232
  hence holo: "f holomorphic_on ball z r - {z}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2233
    by (subst (asm) analytic_on_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2234
  have "eventually (\<lambda>w. w \<in> ball z r - {z}) (at z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2235
    using r by (intro eventually_at_in_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2236
  from freq and this have "frequently (\<lambda>w. f w = 0 \<and> w \<in> ball z r - {z}) (at z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2237
    using frequently_eventually_frequently by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2238
  hence "frequently (\<lambda>w. w \<in> {w\<in>ball z r - {z}. f w = 0}) (at z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2239
    by (simp add: conj_commute)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2240
  hence limpt: "z islimpt {w\<in>ball z r - {z}. f w = 0}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2241
    using islimpt_conv_frequently_at by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2242
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2243
  define g where "g = (\<lambda>w. if w = z then 0 else f w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2244
  have "f \<midarrow>z\<rightarrow> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2245
    by (intro not_essential_frequently_0_imp_tendsto_0 assms)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2246
  hence g_holo: "g holomorphic_on ball z r"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2247
    unfolding g_def by (intro removable_singularity holo) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2248
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2249
  have g_eq_0: "g w = 0" if "w \<in> ball z r" for w
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2250
  proof (rule analytic_continuation[where f = g])
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2251
    show "open (ball z r)" "connected (ball z r)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2252
      using r by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2253
    show "z islimpt {w\<in>ball z r - {z}. f w = 0}"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2254
      by fact
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2255
    show "g w = 0" if "w \<in> {w \<in> ball z r - {z}. f w = 0}" for w
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2256
      using that by (auto simp: g_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2257
  qed (use r that g_holo in auto)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2258
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2259
  have "eventually (\<lambda>w. w \<in> ball z r - {z}) (at z)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2260
    using r by (intro eventually_at_in_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2261
  thus "eventually (\<lambda>w. f w = 0) (at z)"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2262
    by (metis freq non_zero_neighbour not_eventually not_frequently sing)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2263
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2264
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2265
lemma pole_imp_not_constant:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2266
  fixes f :: "'a :: {perfect_space} \<Rightarrow> _"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2267
  assumes "is_pole f x" "open A" "x \<in> A" "A \<subseteq> insert x B"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2268
  shows   "\<not>f constant_on B"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2269
proof
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2270
  assume *: "f constant_on B"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2271
  then obtain c where c: "\<forall>x\<in>B. f x = c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2272
    by (auto simp: constant_on_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2273
  have "eventually (\<lambda>y. y \<in> A - {x}) (at x)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2274
    using assms by (intro eventually_at_in_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2275
  hence "eventually (\<lambda>y. f y = c) (at x)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2276
    by eventually_elim (use c assms in auto)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2277
  hence **: "f \<midarrow>x\<rightarrow> c"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2278
    by (simp add: tendsto_eventually)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2279
  show False
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2280
    using ** \<open>is_pole f x\<close> at_neq_bot is_pole_def 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2281
          not_tendsto_and_filterlim_at_infinity by blast
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2282
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2283
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2284
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2285
lemma neg_zorder_imp_is_pole:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2286
  assumes iso: "isolated_singularity_at f z" and f_ness: "not_essential f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2287
      and "zorder f z < 0" and fre_nz: "\<exists>\<^sub>F w in at z. f w \<noteq> 0 "
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2288
    shows "is_pole f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2289
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2290
  define P where "P = zor_poly f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2291
  define n where "n = zorder f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2292
  have "n<0" unfolding n_def by (simp add: assms(3))
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2293
  define nn where "nn = nat (-n)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2294
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2295
  obtain r where r: "P z \<noteq> 0" "r>0" and r_holo: "P holomorphic_on cball z r" and
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2296
       w_Pn: "(\<forall>w\<in>cball z r - {z}. f w = P w * (w-z) powi n \<and> P w \<noteq> 0)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2297
    using zorder_exist[OF iso f_ness fre_nz,folded P_def n_def] by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2298
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2299
  have "is_pole (\<lambda>w. P w * (w-z) powi n) z"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2300
    unfolding is_pole_def
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2301
  proof (rule tendsto_mult_filterlim_at_infinity)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2302
    show "P \<midarrow>z\<rightarrow> P z"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2303
      by (metis \<open>r>0\<close> r_holo centre_in_ball continuous_on_interior 
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2304
                holomorphic_on_imp_continuous_on interior_cball isContD)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2305
    show "P z\<noteq>0" by (simp add: \<open>P z \<noteq> 0\<close>)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2306
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2307
    have "LIM x at z. inverse ((x - z) ^ nat (-n)) :> at_infinity"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2308
      apply (subst filterlim_inverse_at_iff[symmetric])
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2309
      using \<open>n<0\<close>
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2310
      by (auto intro!:tendsto_eq_intros filterlim_atI
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2311
              simp add: eventually_at_filter)
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  2312
    then show "LIM x at z. (x - z) powi n :> at_infinity"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2313
    proof (elim filterlim_mono_eventually)
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  2314
      have "inverse ((x - z) ^ nat (-n)) = (x - z) powi n"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2315
        if "x\<noteq>z" for x
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  2316
        by (metis \<open>n < 0\<close> linorder_not_le power_int_def power_inverse)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2317
      then show "\<forall>\<^sub>F x in at z. inverse ((x - z) ^ nat (-n))
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  2318
                  = (x - z) powi n"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2319
        by (simp add: eventually_at_filter)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2320
    qed auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2321
  qed
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2322
  moreover have "\<forall>\<^sub>F w in at z. f w =  P w * (w-z) powi n"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2323
    unfolding eventually_at_le
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2324
    using w_Pn \<open>r>0\<close> by (force simp add: dist_commute)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2325
  ultimately show ?thesis using is_pole_cong by fast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2326
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2327
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2328
lemma is_pole_divide_zorder:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2329
  fixes f g:: "complex \<Rightarrow> complex" and z::complex
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2330
  assumes f_iso: "isolated_singularity_at f z" and g_iso: "isolated_singularity_at g z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2331
      and f_ness: "not_essential f z" and g_ness: "not_essential g z"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2332
      and fg_nconst: "\<exists>\<^sub>Fw in (at z). f w * g w\<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2333
      and z_less: "zorder f z < zorder g z"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2334
    shows "is_pole (\<lambda>z. f z / g z) z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2335
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2336
  define fn gn fg where "fn=zorder f z" and "gn=zorder g z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2337
                        and "fg=(\<lambda>w. f w / g w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2338
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2339
  have "isolated_singularity_at fg z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2340
    unfolding fg_def using f_iso g_iso g_ness
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2341
    by (auto intro: singularity_intros)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2342
  moreover have "not_essential fg z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2343
    unfolding fg_def using f_iso g_iso g_ness f_ness
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2344
    by (auto intro: singularity_intros)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2345
  moreover have "zorder fg z < 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2346
  proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2347
    have "zorder fg z = fn - gn"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2348
      using zorder_divide[OF f_iso g_iso f_ness g_ness fg_nconst]
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2349
      by (simp add: fg_def fn_def gn_def) 
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2350
    then show ?thesis
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2351
      using z_less by (simp add: fn_def gn_def)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2352
  qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2353
  moreover have "\<exists>\<^sub>F w in at z. fg w \<noteq> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2354
    using fg_nconst unfolding fg_def by force
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2355
  ultimately show "is_pole fg z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2356
    using neg_zorder_imp_is_pole by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2357
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2358
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2359
lemma isolated_pole_imp_nzero_times:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2360
  assumes f_iso: "isolated_singularity_at f z"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2361
    and "is_pole f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2362
  shows "\<exists>\<^sub>Fw in (at z). deriv f w * f w \<noteq> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2363
proof (rule ccontr)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2364
  assume "\<not> (\<exists>\<^sub>F w in at z.  deriv f w  * f w \<noteq> 0)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2365
  then have "\<forall>\<^sub>F x in at z. deriv f x * f x = 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2366
    unfolding not_frequently by simp
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2367
  moreover have "\<forall>\<^sub>F w in at z. f w \<noteq> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2368
    using non_zero_neighbour_pole[OF \<open>is_pole f z\<close>] .
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2369
  moreover have "\<forall>\<^sub>F w in at z. deriv f w \<noteq> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2370
    using is_pole_deriv[OF \<open>is_pole f z\<close> f_iso,THEN non_zero_neighbour_pole]
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2371
    .
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2372
  ultimately have "\<forall>\<^sub>F w in at z. False"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2373
    by eventually_elim auto
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2374
  then show False by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2375
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2376
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2377
lemma isolated_pole_imp_neg_zorder:
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2378
  assumes "isolated_singularity_at f z" and "is_pole f z"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2379
  shows "zorder f z < 0"
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2380
  using analytic_imp_holomorphic assms centre_in_ball isolated_singularity_at_def zorder_exist_pole by blast
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2381
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2382
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2383
lemma isolated_singularity_at_deriv[singularity_intros]:
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2384
  assumes "isolated_singularity_at f x"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2385
  shows "isolated_singularity_at (deriv f) x"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2386
  by (meson analytic_deriv assms isolated_singularity_at_def)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2387
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2388
lemma zorder_deriv_minus_1:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2389
  fixes f g:: "complex \<Rightarrow> complex" and z::complex
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2390
  assumes f_iso: "isolated_singularity_at f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2391
      and f_ness: "not_essential f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2392
      and f_nconst: "\<exists>\<^sub>F w in at z. f w \<noteq> 0"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2393
      and f_ord: "zorder f z \<noteq>0"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2394
    shows "zorder (deriv f) z = zorder f z - 1"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2395
proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2396
  define P where "P = zor_poly f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2397
  define n where "n = zorder f z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2398
  have "n\<noteq>0" unfolding n_def using f_ord by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2399
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2400
  obtain r where "P z \<noteq> 0" "r>0" and P_holo: "P holomorphic_on cball z r"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2401
          and "(\<forall>w\<in>cball z r - {z}. f w
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2402
                            = P w * (w-z) powi n \<and> P w \<noteq> 0)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2403
    using zorder_exist[OF f_iso f_ness f_nconst,folded P_def n_def] by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2404
  from this(4)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2405
  have f_eq: "(\<forall>w\<in>cball z r - {z}. f w
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2406
                            = P w * (w-z) powi n \<and> P w \<noteq> 0)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2407
    using complex_powr_of_int f_ord n_def by presburger
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2408
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2409
  define D where "D = (\<lambda>w. (deriv P w * (w-z) + of_int n * P w)
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2410
                          * (w-z) powi (n - 1))"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2411
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2412
  have deriv_f_eq: "deriv f w = D w" if "w \<in> ball z r - {z}" for w
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2413
  proof -
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2414
    have ev': "eventually (\<lambda>w. w \<in> ball z r - {z}) (nhds w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2415
      using that by (intro eventually_nhds_in_open) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2416
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2417
    define wz where "wz = w - z"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2418
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2419
    have "wz \<noteq>0" unfolding wz_def using that by auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2420
    moreover have "(P has_field_derivative deriv P w) (at w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2421
      by (meson DiffD1 Elementary_Metric_Spaces.open_ball P_holo
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2422
          ball_subset_cball holomorphic_derivI holomorphic_on_subset that)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2423
    ultimately have "((\<lambda>w. P w * (w-z) powi n) has_field_derivative D w) (at w)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2424
      unfolding D_def using that
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2425
      apply (auto intro!: derivative_eq_intros)
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2426
      by (auto simp: algebra_simps simp flip:power_int_add_1' wz_def)
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2427
    also have "?this \<longleftrightarrow> (f has_field_derivative D w) (at w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2428
      using f_eq
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2429
      by (intro has_field_derivative_cong_ev refl eventually_mono[OF ev']) auto
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2430
    ultimately have "(f has_field_derivative D w) (at w)" by simp
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2431
    moreover have "(f has_field_derivative deriv f w) (at w)"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2432
      by (metis DERIV_imp_deriv calculation)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2433
    ultimately show ?thesis using DERIV_imp_deriv by blast
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2434
  qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2435
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2436
  show "zorder (deriv f) z = n - 1"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2437
  proof (rule zorder_eqI)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2438
    show "open (ball z r)" "z \<in> ball z r"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2439
      using \<open>r > 0\<close> by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2440
    define g where "g=(\<lambda>w. (deriv P w * (w-z) + of_int n * P w))"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2441
    show "g holomorphic_on ball z r"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2442
      unfolding g_def using P_holo
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2443
      by (auto intro!:holomorphic_intros)
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2444
    show "g z \<noteq> 0"
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2445
      unfolding g_def using \<open>P z \<noteq> 0\<close> \<open>n\<noteq>0\<close> by auto
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2446
    show "deriv f w = (deriv P w * (w-z) + of_int n * P w) * (w-z) powi (n - 1)"
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2447
      if "w \<in> ball z r" "w \<noteq> z" for w
77322
9c295f84d55f Replacing z powr of_int i by z powi i and adding new material from the AFP
paulson <lp15@cam.ac.uk>
parents: 77277
diff changeset
  2448
      using D_def deriv_f_eq that by blast
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2449
  qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2450
qed
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2451
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2452
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2453
lemma deriv_divide_is_pole: \<comment>\<open>Generalises @{thm zorder_deriv}\<close>
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2454
  fixes f g:: "complex \<Rightarrow> complex" and z::complex
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2455
  assumes f_iso: "isolated_singularity_at f z"
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2456
      and f_ness: "not_essential f z" 
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2457
      and fg_nconst: "\<exists>\<^sub>Fw in (at z). deriv f w *  f w \<noteq> 0"
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2458
      and f_ord: "zorder f z \<noteq>0"
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2459
    shows "is_pole (\<lambda>z. deriv f z / f z) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2460
proof (rule neg_zorder_imp_is_pole)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2461
  define ff where "ff=(\<lambda>w. deriv f w / f w)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2462
  show "isolated_singularity_at ff z" 
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2463
    using f_iso f_ness unfolding ff_def
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2464
    by (auto intro: singularity_intros)
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2465
  show "not_essential ff z" 
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2466
    unfolding ff_def using f_ness f_iso by (auto intro: singularity_intros)
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2467
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2468
  have "zorder ff z =  zorder (deriv f) z - zorder f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2469
    unfolding ff_def using f_iso f_ness fg_nconst
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2470
    using isolated_singularity_at_deriv not_essential_deriv zorder_divide by blast
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2471
  moreover have "zorder (deriv f) z = zorder f z - 1"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2472
    using f_iso f_ness f_ord fg_nconst frequently_elim1 zorder_deriv_minus_1 by fastforce
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2473
  ultimately show "zorder ff z < 0" by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2474
    
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2475
  show "\<exists>\<^sub>F w in at z. ff w \<noteq> 0" 
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2476
    unfolding ff_def using fg_nconst by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2477
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2478
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2479
lemma is_pole_deriv_divide_is_pole:
81899
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2480
  fixes f g:: "complex \<Rightarrow> complex" and z::complex
1171ea4a23e4 more tidying
paulson <lp15@cam.ac.uk>
parents: 79945
diff changeset
  2481
  assumes f_iso: "isolated_singularity_at f z"
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2482
      and "is_pole f z" 
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2483
    shows "is_pole (\<lambda>z. deriv f z / f z) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2484
proof (rule deriv_divide_is_pole[OF f_iso])
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2485
  show "not_essential f z" 
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2486
    using \<open>is_pole f z\<close> unfolding not_essential_def by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2487
  show "\<exists>\<^sub>F w in at z. deriv f w * f w \<noteq> 0"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2488
    using assms f_iso isolated_pole_imp_nzero_times by blast
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2489
  show "zorder f z \<noteq> 0"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2490
    using isolated_pole_imp_neg_zorder assms by fastforce
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2491
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2492
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2493
subsection \<open>Isolated zeroes\<close>
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2494
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2495
definition isolated_zero :: "(complex \<Rightarrow> complex) \<Rightarrow> complex \<Rightarrow> bool" where
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2496
  "isolated_zero f z \<longleftrightarrow> f z = 0 \<and> eventually (\<lambda>z. f z \<noteq> 0) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2497
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2498
lemma isolated_zero_altdef: "isolated_zero f z \<longleftrightarrow> f z = 0 \<and> \<not>z islimpt {z. f z = 0}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2499
  unfolding isolated_zero_def eventually_at_filter eventually_nhds islimpt_def by blast
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2500
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2501
lemma isolated_zero_mult1:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2502
  assumes "isolated_zero f x" "isolated_zero g x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2503
  shows   "isolated_zero (\<lambda>x. f x * g x) x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2504
proof -
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2505
  have "\<forall>\<^sub>F x in at x. f x \<noteq> 0" "\<forall>\<^sub>F x in at x. g x \<noteq> 0"
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2506
    using assms unfolding isolated_zero_def by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2507
  hence "eventually (\<lambda>x. f x * g x \<noteq> 0) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2508
    by eventually_elim auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2509
  with assms show ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2510
    by (auto simp: isolated_zero_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2511
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2512
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2513
lemma isolated_zero_mult2:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2514
  assumes "isolated_zero f x" "g x \<noteq> 0" "g analytic_on {x}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2515
  shows   "isolated_zero (\<lambda>x. f x * g x) x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2516
proof -
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2517
  have "eventually (\<lambda>x. f x \<noteq> 0) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2518
    using assms unfolding isolated_zero_def by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2519
  moreover have "eventually (\<lambda>x. g x \<noteq> 0) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2520
    using analytic_at_neq_imp_eventually_neq[of g x 0] assms by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2521
  ultimately have "eventually (\<lambda>x. f x * g x \<noteq> 0) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2522
    by eventually_elim auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2523
  thus ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2524
    using assms(1) by (auto simp: isolated_zero_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2525
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2526
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2527
lemma isolated_zero_mult3:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2528
  assumes "isolated_zero f x" "g x \<noteq> 0" "g analytic_on {x}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2529
  shows   "isolated_zero (\<lambda>x. g x * f x) x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2530
  using isolated_zero_mult2[OF assms] by (simp add: mult_ac)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2531
  
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2532
lemma isolated_zero_prod:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2533
  assumes "\<And>x. x \<in> I \<Longrightarrow> isolated_zero (f x) z" "I \<noteq> {}" "finite I"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2534
  shows   "isolated_zero (\<lambda>y. \<Prod>x\<in>I. f x y) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2535
  using assms(3,2,1) by (induction rule: finite_ne_induct) (auto intro: isolated_zero_mult1)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2536
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2537
lemma non_isolated_zero':
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2538
  assumes "isolated_singularity_at f z" "not_essential f z" "f z = 0" "\<not>isolated_zero f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2539
  shows   "eventually (\<lambda>z. f z = 0) (at z)"
78517
28c1f4f5335f Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents: 77322
diff changeset
  2540
  by (metis assms isolated_zero_def non_zero_neighbour not_eventually)
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2541
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2542
lemma non_isolated_zero:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2543
  assumes "\<not>isolated_zero f z" "f analytic_on {z}" "f z = 0"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2544
  shows   "eventually (\<lambda>z. f z = 0) (nhds z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2545
proof -
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2546
  have "eventually (\<lambda>z. f z = 0) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2547
    by (rule non_isolated_zero')
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2548
       (use assms in \<open>auto intro: not_essential_analytic isolated_singularity_at_analytic\<close>)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2549
  with \<open>f z = 0\<close> show ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2550
    unfolding eventually_at_filter by (auto elim!: eventually_mono)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2551
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2552
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2553
lemma not_essential_compose:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2554
  assumes "not_essential f (g z)" "g analytic_on {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2555
  shows   "not_essential (\<lambda>x. f (g x)) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2556
proof (cases "isolated_zero (\<lambda>w. g w - g z) z")
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2557
  case False
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2558
  hence "eventually (\<lambda>w. g w - g z = 0) (nhds z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2559
    by (rule non_isolated_zero) (use assms in \<open>auto intro!: analytic_intros\<close>)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2560
  hence "not_essential (\<lambda>x. f (g x)) z \<longleftrightarrow> not_essential (\<lambda>_. f (g z)) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2561
    by (intro not_essential_cong refl)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2562
       (auto elim!: eventually_mono simp: eventually_at_filter)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2563
  thus ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2564
    by (simp add: not_essential_const)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2565
next
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2566
  case True
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2567
  hence ev: "eventually (\<lambda>w. g w \<noteq> g z) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2568
    by (auto simp: isolated_zero_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2569
  from assms consider c where "f \<midarrow>g z\<rightarrow> c" | "is_pole f (g z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2570
    by (auto simp: not_essential_def)  
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2571
  have "isCont g z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2572
    by (rule analytic_at_imp_isCont) fact
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2573
  hence lim: "g \<midarrow>z\<rightarrow> g z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2574
    using isContD by blast
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2575
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2576
  from assms(1) consider c where "f \<midarrow>g z\<rightarrow> c" | "is_pole f (g z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2577
    unfolding not_essential_def by blast
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2578
  thus ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2579
  proof cases
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2580
    fix c assume "f \<midarrow>g z\<rightarrow> c"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2581
    hence "(\<lambda>x. f (g x)) \<midarrow>z\<rightarrow> c"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2582
      by (rule filterlim_compose) (use lim ev in \<open>auto simp: filterlim_at\<close>)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2583
    thus ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2584
      by (auto simp: not_essential_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2585
  next
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2586
    assume "is_pole f (g z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2587
    hence "is_pole (\<lambda>x. f (g x)) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2588
      by (rule is_pole_compose) fact+
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2589
    thus ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2590
      by (auto simp: not_essential_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2591
  qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2592
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2593
  
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2594
subsection \<open>Isolated points\<close>
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2595
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2596
definition isolated_points_of :: "complex set \<Rightarrow> complex set" where
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2597
  "isolated_points_of A = {z\<in>A. eventually (\<lambda>w. w \<notin> A) (at z)}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2598
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2599
lemma isolated_points_of_altdef: "isolated_points_of A = {z\<in>A. \<not>z islimpt A}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2600
  unfolding isolated_points_of_def islimpt_def eventually_at_filter eventually_nhds by blast
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2601
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2602
lemma isolated_points_of_empty [simp]: "isolated_points_of {} = {}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2603
  and isolated_points_of_UNIV [simp]:  "isolated_points_of UNIV = {}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2604
  by (auto simp: isolated_points_of_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2605
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2606
lemma isolated_points_of_open_is_empty [simp]: "open A \<Longrightarrow> isolated_points_of A = {}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2607
  unfolding isolated_points_of_altdef 
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2608
  by (simp add: interior_limit_point interior_open)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2609
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2610
lemma isolated_points_of_subset: "isolated_points_of A \<subseteq> A"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2611
  by (auto simp: isolated_points_of_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2612
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2613
lemma isolated_points_of_discrete:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2614
  assumes "discrete A"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2615
  shows   "isolated_points_of A = A"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2616
  using assms by (auto simp: isolated_points_of_def discrete_altdef)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2617
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2618
lemmas uniform_discreteI1 = uniformI1
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2619
lemmas uniform_discreteI2 = uniformI2
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2620
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2621
lemma isolated_singularity_at_compose:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2622
  assumes "isolated_singularity_at f (g z)" "g analytic_on {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2623
  shows   "isolated_singularity_at (\<lambda>x. f (g x)) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2624
proof (cases "isolated_zero (\<lambda>w. g w - g z) z")
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2625
  case False
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2626
  hence "eventually (\<lambda>w. g w - g z = 0) (nhds z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2627
    by (rule non_isolated_zero) (use assms in \<open>auto intro!: analytic_intros\<close>)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2628
  hence "isolated_singularity_at (\<lambda>x. f (g x)) z \<longleftrightarrow> isolated_singularity_at (\<lambda>_. f (g z)) z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2629
    by (intro isolated_singularity_at_cong refl)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2630
       (auto elim!: eventually_mono simp: eventually_at_filter)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2631
  thus ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2632
    by (simp add: isolated_singularity_at_const)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2633
next
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2634
  case True
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2635
  from assms(1) obtain r where r: "r > 0" "f analytic_on ball (g z) r - {g z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2636
    by (auto simp: isolated_singularity_at_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2637
  hence holo_f: "f holomorphic_on ball (g z) r - {g z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2638
    by (subst (asm) analytic_on_open) auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2639
  from assms(2) obtain r' where r': "r' > 0" "g holomorphic_on ball z r'"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2640
    by (auto simp: analytic_on_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2641
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2642
  have "continuous_on (ball z r') g"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2643
    using holomorphic_on_imp_continuous_on r' by blast
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2644
  hence "isCont g z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2645
    using r' by (subst (asm) continuous_on_eq_continuous_at) auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2646
  hence "g \<midarrow>z\<rightarrow> g z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2647
    using isContD by blast
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2648
  hence "eventually (\<lambda>w. g w \<in> ball (g z) r) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2649
    using \<open>r > 0\<close> unfolding tendsto_def by force
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2650
  moreover have "eventually (\<lambda>w. g w \<noteq> g z) (at z)" using True
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2651
    by (auto simp: isolated_zero_def elim!: eventually_mono)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2652
  ultimately have "eventually (\<lambda>w. g w \<in> ball (g z) r - {g z}) (at z)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2653
    by eventually_elim auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2654
  then obtain r'' where r'': "r'' > 0" "\<forall>w\<in>ball z r''-{z}. g w \<in> ball (g z) r - {g z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2655
    unfolding eventually_at_filter eventually_nhds_metric ball_def
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2656
    by (auto simp: dist_commute)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2657
  have "f \<circ> g holomorphic_on ball z (min r' r'') - {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2658
  proof (rule holomorphic_on_compose_gen)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2659
    show "g holomorphic_on ball z (min r' r'') - {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2660
      by (rule holomorphic_on_subset[OF r'(2)]) auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2661
    show "f holomorphic_on ball (g z) r - {g z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2662
      by fact
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2663
    show "g ` (ball z (min r' r'') - {z}) \<subseteq> ball (g z) r - {g z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2664
      using r'' by force
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2665
  qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2666
  hence "f \<circ> g analytic_on ball z (min r' r'') - {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2667
    by (subst analytic_on_open) auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2668
  thus ?thesis using \<open>r' > 0\<close> \<open>r'' > 0\<close>
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2669
    by (auto simp: isolated_singularity_at_def o_def intro!: exI[of _ "min r' r''"])
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2670
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2671
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2672
lemma is_pole_power_int_0:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2673
  assumes "f analytic_on {x}" "isolated_zero f x" "n < 0"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2674
  shows   "is_pole (\<lambda>x. f x powi n) x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2675
proof -
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2676
  have "f \<midarrow>x\<rightarrow> f x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2677
    using assms(1) by (simp add: analytic_at_imp_isCont isContD)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2678
  with assms show ?thesis
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2679
    unfolding is_pole_def
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2680
    by (intro filterlim_power_int_neg_at_infinity) (auto simp: isolated_zero_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2681
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2682
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2683
lemma isolated_zero_imp_not_constant_on:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2684
  assumes "isolated_zero f x" "x \<in> A" "open A"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2685
  shows   "\<not>f constant_on A"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2686
proof
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2687
  assume "f constant_on A"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2688
  then obtain c where c: "\<And>x. x \<in> A \<Longrightarrow> f x = c"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2689
    by (auto simp: constant_on_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2690
  from assms and c[of x] have [simp]: "c = 0"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2691
    by (auto simp: isolated_zero_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2692
  have "eventually (\<lambda>x. f x \<noteq> 0) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2693
    using assms by (auto simp: isolated_zero_def)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2694
  moreover have "eventually (\<lambda>x. x \<in> A) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2695
    using assms by (intro eventually_at_in_open') auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2696
  ultimately have "eventually (\<lambda>x. False) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2697
    by eventually_elim (use c in auto)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2698
  thus False
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2699
    by simp
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2700
qed
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77223
diff changeset
  2701
77223
607e1e345e8f Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents: 76900
diff changeset
  2702
end