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