author | nipkow |
Tue, 17 Jun 2025 14:11:40 +0200 | |
changeset 82733 | 8b537e1af2ec |
parent 78517 | 28c1f4f5335f |
permissions | -rw-r--r-- |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1 |
section \<open>The Residue Theorem, the Argument Principle and Rouch\'{e}'s Theorem\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
2 |
theory Residue_Theorem |
73048
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
3 |
imports Complex_Residues "HOL-Library.Landau_Symbols" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
4 |
begin |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
5 |
|
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
|
6 |
text \<open>Several theorems that could be moved up, |
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
|
7 |
IF there were a previous theory importing both Landau Symbols and Elementary Metric Spaces\<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
|
8 |
|
77277
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
9 |
lemma continuous_bounded_at_infinity_imp_bounded: |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
10 |
fixes f :: "real \<Rightarrow> 'a :: real_normed_field" |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
11 |
assumes "f \<in> O[at_bot](\<lambda>_. 1)" |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
12 |
assumes "f \<in> O[at_top](\<lambda>_. 1)" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
13 |
assumes cf: "continuous_on UNIV f" |
77277
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
14 |
shows "bounded (range f)" |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
15 |
proof - |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
16 |
obtain c1 c2 |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
17 |
where "eventually (\<lambda>x. norm (f x) \<le> c1) at_bot" "eventually (\<lambda>x. norm (f x) \<le> c2) at_top" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
18 |
using assms by (auto elim!: landau_o.bigE) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
19 |
then obtain x1 x2 where x1: "\<And>x. x \<le> x1 \<Longrightarrow> norm (f x) \<le> c1" and x2: "\<And>x. x \<ge> x2 \<Longrightarrow> norm (f x) \<le> c2" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
20 |
by (auto simp: eventually_at_bot_linorder eventually_at_top_linorder) |
77277
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
21 |
have "compact (f ` {x1..x2})" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
22 |
by (intro compact_continuous_image continuous_on_subset[OF cf]) auto |
77277
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
23 |
hence "bounded (f ` {x1..x2})" |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
24 |
by (rule compact_imp_bounded) |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
25 |
then obtain c3 where c3: "\<And>x. x \<in> {x1..x2} \<Longrightarrow> norm (f x) \<le> c3" |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
26 |
unfolding bounded_iff by fast |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
27 |
have "norm (f x) \<le> Max {c1, c2, c3}" for x |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
28 |
by (cases "x \<le> x1"; cases "x \<ge> x2") (use x1 x2 c3 in \<open>auto simp: le_max_iff_disj\<close>) |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
29 |
thus ?thesis |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
30 |
unfolding bounded_iff by blast |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
31 |
qed |
c6b50597abbc
More of Eberl's contributions: memomorphic functions
paulson <lp15@cam.ac.uk>
parents:
77223
diff
changeset
|
32 |
|
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
|
33 |
lemma holomorphic_on_extend: |
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
|
34 |
assumes "f holomorphic_on S - {\<xi>}" "\<xi> \<in> interior S" "f \<in> O[at \<xi>](\<lambda>_. 1)" |
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
|
35 |
shows "(\<exists>g. g holomorphic_on S \<and> (\<forall>z\<in>S - {\<xi>}. g z = f 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
|
36 |
by (subst holomorphic_on_extend_bounded) (insert assms, auto elim!: landau_o.bigE) |
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
|
37 |
|
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
|
38 |
lemma removable_singularities: |
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
|
39 |
assumes "finite X" "X \<subseteq> interior S" "f holomorphic_on (S - X)" |
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
|
40 |
assumes "\<And>z. z \<in> X \<Longrightarrow> f \<in> O[at z](\<lambda>_. 1)" |
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
|
41 |
shows "\<exists>g. g holomorphic_on S \<and> (\<forall>z\<in>S-X. g z = f 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
|
42 |
using assms |
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
|
43 |
proof (induction arbitrary: f rule: finite_induct) |
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
|
44 |
case empty |
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
|
45 |
thus ?case by auto |
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
|
46 |
next |
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
|
47 |
case (insert z0 X f) |
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
|
48 |
from insert.prems and insert.hyps have z0: "z0 \<in> interior (S - X)" |
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
|
49 |
by (auto simp: interior_diff finite_imp_closed) |
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
|
50 |
hence "\<exists>g. g holomorphic_on (S - X) \<and> (\<forall>z\<in>S - X - {z0}. g z = f 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
|
51 |
using insert.prems insert.hyps by (intro holomorphic_on_extend) auto |
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
|
52 |
then obtain g where g: "g holomorphic_on (S - X)" "\<forall>z\<in>S - X - {z0}. g z = f z" by blast |
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
|
53 |
have "\<exists>h. h holomorphic_on S \<and> (\<forall>z\<in>S - X. h z = g 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
|
54 |
proof (rule insert.IH) |
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
|
55 |
fix z0' assume z0': "z0' \<in> X" |
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
|
56 |
hence "eventually (\<lambda>z. z \<in> interior S - (X - {z0'}) - {z0}) (nhds 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
|
57 |
using insert.prems insert.hyps |
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
|
58 |
by (intro eventually_nhds_in_open open_Diff finite_imp_closed) auto |
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
|
59 |
hence ev: "eventually (\<lambda>z. z \<in> S - X - {z0}) (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
|
60 |
unfolding eventually_at_filter |
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
|
61 |
by eventually_elim (insert z0' insert.hyps interior_subset[of S], auto) |
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
|
62 |
have "g \<in> \<Theta>[at z0'](f)" |
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
|
63 |
by (intro bigthetaI_cong eventually_mono[OF ev]) (insert g, auto) |
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
|
64 |
also have "f \<in> O[at z0'](\<lambda>_. 1)" |
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
|
65 |
using z0' by (intro insert.prems) auto |
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
|
66 |
finally show "g \<in> \<dots>" . |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
67 |
qed (use insert.prems g in 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
|
68 |
then obtain h where "h holomorphic_on S" "\<forall>z\<in>S - X. h z = g z" by blast |
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
|
69 |
with g have "h holomorphic_on S" "\<forall>z\<in>S - insert z0 X. h z = f z" by auto |
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
|
70 |
thus ?case by blast |
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
|
71 |
qed |
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
|
72 |
|
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
|
73 |
lemma continuous_imp_bigo_1: |
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
|
74 |
assumes "continuous (at x within A) f" |
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
|
75 |
shows "f \<in> O[at x within A](\<lambda>_. 1)" |
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
|
76 |
proof (rule bigoI_tendsto) |
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
|
77 |
from assms show "((\<lambda>x. f x / 1) \<longlongrightarrow> f x) (at x within A)" |
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
|
78 |
by (auto simp: continuous_within) |
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
|
79 |
qed auto |
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
|
80 |
|
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
|
81 |
lemma taylor_bigo_linear: |
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
|
82 |
assumes "f field_differentiable at x0 within A" |
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
|
83 |
shows "(\<lambda>x. f x - f x0) \<in> O[at x0 within A](\<lambda>x. x - x0)" |
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
|
84 |
proof - |
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
|
85 |
from assms obtain f' where "(f has_field_derivative f') (at x0 within A)" |
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
|
86 |
by (auto simp: field_differentiable_def) |
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
|
87 |
hence "((\<lambda>x. (f x - f x0) / (x - x0)) \<longlongrightarrow> f') (at x0 within A)" |
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
|
88 |
by (auto simp: has_field_derivative_iff) |
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
|
89 |
thus ?thesis by (intro bigoI_tendsto[where c = f']) (auto simp: eventually_at_filter) |
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
|
90 |
qed |
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
|
91 |
|
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
|
92 |
|
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
93 |
subsection \<open>Cauchy's residue theorem\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
94 |
|
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
95 |
lemma get_integrable_path: |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
96 |
assumes "open S" "connected (S-pts)" "finite pts" "f holomorphic_on (S-pts) " "a\<in>S-pts" "b\<in>S-pts" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
97 |
obtains g where "valid_path g" "pathstart g = a" "pathfinish g = b" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
98 |
"path_image g \<subseteq> S-pts" "f contour_integrable_on g" using assms |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
99 |
proof (induct arbitrary:S thesis a rule:finite_induct[OF \<open>finite pts\<close>]) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
100 |
case 1 |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
101 |
obtain g where "valid_path g" "path_image g \<subseteq> S" "pathstart g = a" "pathfinish g = b" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
102 |
using connected_open_polynomial_connected[OF \<open>open S\<close>,of a b ] \<open>connected (S - {})\<close> |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
103 |
valid_path_polynomial_function "1.prems"(6) "1.prems"(7) by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
104 |
moreover have "f contour_integrable_on g" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
105 |
using contour_integrable_holomorphic_simple[OF _ \<open>open S\<close> \<open>valid_path g\<close> \<open>path_image g \<subseteq> S\<close>,of f] |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
106 |
\<open>f holomorphic_on S - {}\<close> |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
107 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
108 |
ultimately show ?case using "1"(1)[of g] by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
109 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
110 |
case idt:(2 p pts) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
111 |
obtain e where "e>0" and e:"\<forall>w\<in>ball a e. w \<in> S \<and> (w \<noteq> a \<longrightarrow> w \<notin> insert p pts)" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
112 |
using finite_ball_avoid[OF \<open>open S\<close> \<open>finite (insert p pts)\<close>, of a] |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
113 |
\<open>a \<in> S - insert p pts\<close> |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
114 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
115 |
define a' where "a' \<equiv> a+e/2" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
116 |
have "a'\<in>S-{p} -pts" using e[rule_format,of "a+e/2"] \<open>e>0\<close> |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
117 |
by (auto simp add:dist_complex_def a'_def) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
118 |
then obtain g' where g'[simp]:"valid_path g'" "pathstart g' = a'" "pathfinish g' = b" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
119 |
"path_image g' \<subseteq> S - {p} - pts" "f contour_integrable_on g'" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
120 |
using idt.hyps(3)[of a' "S-{p}"] idt.prems idt.hyps(1) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
121 |
by (metis Diff_insert2 open_delete) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
122 |
define g where "g \<equiv> linepath a a' +++ g'" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
123 |
have "valid_path g" unfolding g_def by (auto intro: valid_path_join) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
124 |
moreover have "pathstart g = a" and "pathfinish g = b" unfolding g_def by auto |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
125 |
moreover have "path_image g \<subseteq> S - insert p pts" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
126 |
unfolding g_def |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
127 |
proof (rule subset_path_image_join) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
128 |
have "closed_segment a a' \<subseteq> ball a e" using \<open>e>0\<close> |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
129 |
by (auto dest!:segment_bound1 simp:a'_def dist_complex_def norm_minus_commute) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
130 |
then show "path_image (linepath a a') \<subseteq> S - insert p pts" using e idt(9) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
131 |
by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
132 |
next |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
133 |
show "path_image g' \<subseteq> S - insert p pts" using g'(4) by blast |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
134 |
qed |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
135 |
moreover have "f contour_integrable_on g" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
136 |
proof - |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
137 |
have "closed_segment a a' \<subseteq> ball a e" using \<open>e>0\<close> |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
138 |
by (auto dest!:segment_bound1 simp:a'_def dist_complex_def norm_minus_commute) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
139 |
then have "closed_segment a a' \<subseteq> S - insert p pts" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
140 |
using e idt.prems(6) by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
141 |
then have "continuous_on (closed_segment a a') f" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
142 |
using holomorphic_on_imp_continuous_on holomorphic_on_subset idt.prems(5) by presburger |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
143 |
then show ?thesis |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
144 |
using contour_integrable_continuous_linepath by (simp add: g_def) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
145 |
qed |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
146 |
ultimately show ?case using idt.prems(1)[of g] by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
147 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
148 |
|
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
149 |
lemma Cauchy_theorem_aux: |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
150 |
assumes "open S" "connected (S-pts)" "finite pts" "pts \<subseteq> S" "f holomorphic_on S-pts" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
151 |
"valid_path g" "pathfinish g = pathstart g" "path_image g \<subseteq> S-pts" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
152 |
"\<forall>z. (z \<notin> S) \<longrightarrow> winding_number g z = 0" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
153 |
"\<forall>p\<in>S. h p>0 \<and> (\<forall>w\<in>cball p (h p). w\<in>S \<and> (w\<noteq>p \<longrightarrow> w \<notin> pts))" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
154 |
shows "contour_integral g f = (\<Sum>p\<in>pts. winding_number g p * contour_integral (circlepath p (h p)) f)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
155 |
using assms |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
156 |
proof (induct arbitrary:S g rule:finite_induct[OF \<open>finite pts\<close>]) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
157 |
case 1 |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
158 |
then show ?case by (simp add: Cauchy_theorem_global contour_integral_unique) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
159 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
160 |
case (2 p pts) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
161 |
note fin[simp] = \<open>finite (insert p pts)\<close> |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
162 |
and connected = \<open>connected (S - insert p pts)\<close> |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
163 |
and valid[simp] = \<open>valid_path g\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
164 |
and g_loop[simp] = \<open>pathfinish g = pathstart g\<close> |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
165 |
and holo[simp]= \<open>f holomorphic_on S - insert p pts\<close> |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
166 |
and path_img = \<open>path_image g \<subseteq> S - insert p pts\<close> |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
167 |
and winding = \<open>\<forall>z. z \<notin> S \<longrightarrow> winding_number g z = 0\<close> |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
168 |
and h = \<open>\<forall>pa\<in>S. 0 < h pa \<and> (\<forall>w\<in>cball pa (h pa). w \<in> S \<and> (w \<noteq> pa \<longrightarrow> w \<notin> insert p pts))\<close> |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
169 |
have "h p>0" and "p\<in>S" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
170 |
and h_p: "\<forall>w\<in>cball p (h p). w \<in> S \<and> (w \<noteq> p \<longrightarrow> w \<notin> insert p pts)" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
171 |
using h \<open>insert p pts \<subseteq> S\<close> by auto |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
172 |
obtain pg where pg[simp]: "valid_path pg" "pathstart pg = pathstart g" "pathfinish pg=p+h p" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
173 |
"path_image pg \<subseteq> S-insert p pts" "f contour_integrable_on pg" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
174 |
proof - |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
175 |
have "p + h p\<in>cball p (h p)" using h[rule_format,of p] |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
176 |
by (simp add: \<open>p \<in> S\<close> dist_norm) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
177 |
then have "p + h p \<in> S - insert p pts" using h[rule_format,of p] \<open>insert p pts \<subseteq> S\<close> |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
178 |
by fastforce |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
179 |
moreover have "pathstart g \<in> S - insert p pts " using path_img by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
180 |
ultimately show ?thesis |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
181 |
using get_integrable_path[OF \<open>open S\<close> connected fin holo,of "pathstart g" "p+h p"] that |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
182 |
by blast |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
183 |
qed |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
184 |
obtain n::int where "n=winding_number g p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
185 |
using integer_winding_number[OF _ g_loop,of p] valid path_img |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
186 |
by (metis DiffD2 Ints_cases insertI1 subset_eq valid_path_imp_path) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
187 |
define p_circ where "p_circ \<equiv> circlepath p (h p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
188 |
define p_circ_pt where "p_circ_pt \<equiv> linepath (p+h p) (p+h p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
189 |
define n_circ where "n_circ \<equiv> \<lambda>n. ((+++) p_circ ^^ n) p_circ_pt" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
190 |
define cp where "cp \<equiv> if n\<ge>0 then reversepath (n_circ (nat n)) else n_circ (nat (- n))" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
191 |
|
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
192 |
have n_circ:"valid_path (n_circ k)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
193 |
"winding_number (n_circ k) p = k" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
194 |
"pathstart (n_circ k) = p + h p" "pathfinish (n_circ k) = p + h p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
195 |
"path_image (n_circ k) = (if k=0 then {p + h p} else sphere p (h p))" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
196 |
"p \<notin> path_image (n_circ k)" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
197 |
"\<And>p'. p'\<notin>S - pts \<Longrightarrow> winding_number (n_circ k) p'=0 \<and> p'\<notin>path_image (n_circ k)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
198 |
"f contour_integrable_on (n_circ k)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
199 |
"contour_integral (n_circ k) f = k * contour_integral p_circ f" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
200 |
for k |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
201 |
proof (induct k) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
202 |
case 0 |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
203 |
show "valid_path (n_circ 0)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
204 |
and "path_image (n_circ 0) = (if 0=0 then {p + h p} else sphere p (h p))" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
205 |
and "winding_number (n_circ 0) p = of_nat 0" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
206 |
and "pathstart (n_circ 0) = p + h p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
207 |
and "pathfinish (n_circ 0) = p + h p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
208 |
and "p \<notin> path_image (n_circ 0)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
209 |
unfolding n_circ_def p_circ_pt_def using \<open>h p > 0\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
210 |
by (auto simp add: dist_norm) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
211 |
show "winding_number (n_circ 0) p'=0 \<and> p'\<notin>path_image (n_circ 0)" when "p'\<notin>S- pts" for p' |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
212 |
unfolding n_circ_def p_circ_pt_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
213 |
apply (auto intro!:winding_number_trivial) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
214 |
by (metis Diff_iff pathfinish_in_path_image pg(3) pg(4) subsetCE subset_insertI that)+ |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
215 |
show "f contour_integrable_on (n_circ 0)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
216 |
unfolding n_circ_def p_circ_pt_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
217 |
by (auto intro!:contour_integrable_continuous_linepath simp add:continuous_on_sing) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
218 |
show "contour_integral (n_circ 0) f = of_nat 0 * contour_integral p_circ f" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
219 |
unfolding n_circ_def p_circ_pt_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
220 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
221 |
case (Suc k) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
222 |
have n_Suc:"n_circ (Suc k) = p_circ +++ n_circ k" unfolding n_circ_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
223 |
have pcirc:"p \<notin> path_image p_circ" "valid_path p_circ" "pathfinish p_circ = pathstart (n_circ k)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
224 |
using Suc(3) unfolding p_circ_def using \<open>h p > 0\<close> by (auto simp add: p_circ_def) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
225 |
have pcirc_image:"path_image p_circ \<subseteq> S - insert p pts" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
226 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
227 |
have "path_image p_circ \<subseteq> cball p (h p)" using \<open>0 < h p\<close> p_circ_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
228 |
then show ?thesis using h_p pcirc(1) by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
229 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
230 |
have pcirc_integrable:"f contour_integrable_on p_circ" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
231 |
by (auto simp add:p_circ_def intro!: pcirc_image[unfolded p_circ_def] |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
232 |
contour_integrable_continuous_circlepath holomorphic_on_imp_continuous_on |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
233 |
holomorphic_on_subset[OF holo]) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
234 |
show "valid_path (n_circ (Suc k))" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
235 |
using valid_path_join[OF pcirc(2) Suc(1) pcirc(3)] unfolding n_circ_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
236 |
show "path_image (n_circ (Suc k)) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
237 |
= (if Suc k = 0 then {p + complex_of_real (h p)} else sphere p (h p))" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
238 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
239 |
have "path_image p_circ = sphere p (h p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
240 |
unfolding p_circ_def using \<open>0 < h p\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
241 |
then show ?thesis unfolding n_Suc using Suc.hyps(5) \<open>h p>0\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
242 |
by (auto simp add: path_image_join[OF pcirc(3)] dist_norm) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
243 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
244 |
then show "p \<notin> path_image (n_circ (Suc k))" using \<open>h p>0\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
245 |
show "winding_number (n_circ (Suc k)) p = of_nat (Suc k)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
246 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
247 |
have "winding_number p_circ p = 1" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
248 |
by (simp add: \<open>h p > 0\<close> p_circ_def winding_number_circlepath_centre) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
249 |
moreover have "p \<notin> path_image (n_circ k)" using Suc(5) \<open>h p>0\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
250 |
then have "winding_number (p_circ +++ n_circ k) p |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
251 |
= winding_number p_circ p + winding_number (n_circ k) p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
252 |
using valid_path_imp_path Suc.hyps(1) Suc.hyps(2) pcirc |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
253 |
apply (intro winding_number_join) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
254 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
255 |
ultimately show ?thesis using Suc(2) unfolding n_circ_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
256 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
257 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
258 |
show "pathstart (n_circ (Suc k)) = p + h p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
259 |
by (simp add: n_circ_def p_circ_def) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
260 |
show "pathfinish (n_circ (Suc k)) = p + h p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
261 |
using Suc(4) unfolding n_circ_def by auto |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
262 |
show "winding_number (n_circ (Suc k)) p'=0 \<and> p'\<notin>path_image (n_circ (Suc k))" when "p'\<notin>S-pts" for p' |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
263 |
proof - |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
264 |
have " p' \<notin> path_image p_circ" using \<open>p \<in> S\<close> h p_circ_def that using pcirc_image by blast |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
265 |
moreover have "p' \<notin> path_image (n_circ k)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
266 |
using Suc.hyps(7) that by blast |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
267 |
moreover have "winding_number p_circ p' = 0" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
268 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
269 |
have "path_image p_circ \<subseteq> cball p (h p)" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
270 |
using h unfolding p_circ_def using \<open>p \<in> S\<close> by fastforce |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
271 |
moreover have "p'\<notin>cball p (h p)" using \<open>p \<in> S\<close> h that "2.hyps"(2) by fastforce |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
272 |
ultimately show ?thesis |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
273 |
unfolding p_circ_def |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
274 |
by (intro winding_number_zero_outside) auto |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
275 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
276 |
ultimately show ?thesis |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
277 |
unfolding n_Suc using Suc.hyps pcirc |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
278 |
by (metis add.right_neutral not_in_path_image_join that valid_path_imp_path winding_number_join) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
279 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
280 |
show "f contour_integrable_on (n_circ (Suc k))" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
281 |
unfolding n_Suc |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
282 |
by (rule contour_integrable_joinI[OF pcirc_integrable Suc(8) pcirc(2) Suc(1)]) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
283 |
show "contour_integral (n_circ (Suc k)) f = (Suc k) * contour_integral p_circ f" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
284 |
by (simp add: Rings.ring_distribs(2) Suc.hyps n_Suc pcirc pcirc_integrable) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
285 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
286 |
have cp[simp]:"pathstart cp = p + h p" "pathfinish cp = p + h p" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
287 |
"valid_path cp" "path_image cp \<subseteq> S - insert p pts" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
288 |
"winding_number cp p = - n" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
289 |
"\<And>p'. p'\<notin>S - pts \<Longrightarrow> winding_number cp p'=0 \<and> p' \<notin> path_image cp" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
290 |
"f contour_integrable_on cp" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
291 |
"contour_integral cp f = - n * contour_integral p_circ f" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
292 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
293 |
show "pathstart cp = p + h p" and "pathfinish cp = p + h p" and "valid_path cp" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
294 |
using n_circ unfolding cp_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
295 |
next |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
296 |
have "sphere p (h p) \<subseteq> S - insert p pts" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
297 |
using h[rule_format,of p] \<open>insert p pts \<subseteq> S\<close> by force |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
298 |
moreover have "p + complex_of_real (h p) \<in> S - insert p pts" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
299 |
using pg(3) pg(4) by (metis pathfinish_in_path_image subsetCE) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
300 |
ultimately show "path_image cp \<subseteq> S - insert p pts" unfolding cp_def |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
301 |
using n_circ(5) by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
302 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
303 |
show "winding_number cp p = - n" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
304 |
unfolding cp_def using winding_number_reversepath n_circ \<open>h p>0\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
305 |
by (auto simp: valid_path_imp_path) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
306 |
next |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
307 |
show "winding_number cp p'=0 \<and> p' \<notin> path_image cp" when "p'\<notin>S - pts" for p' |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
308 |
proof - |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
309 |
have "winding_number (reversepath (n_circ (nat n))) p' = 0" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
310 |
using n_circ that |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
311 |
by (metis add.inverse_neutral valid_path_imp_path winding_number_reversepath) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
312 |
then show ?thesis |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
313 |
using cp_def n_circ(7) that by force |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
314 |
qed |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
315 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
316 |
show "f contour_integrable_on cp" unfolding cp_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
317 |
using contour_integrable_reversepath_eq n_circ(1,8) by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
318 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
319 |
show "contour_integral cp f = - n * contour_integral p_circ f" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
320 |
unfolding cp_def using contour_integral_reversepath[OF n_circ(1)] n_circ(9) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
321 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
322 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
323 |
define g' where "g' \<equiv> g +++ pg +++ cp +++ (reversepath pg)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
324 |
have "contour_integral g' f = (\<Sum>p\<in>pts. winding_number g' p * contour_integral (circlepath p (h p)) f)" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
325 |
proof (rule "2.hyps"(3)[of "S-{p}" "g'",OF _ _ \<open>finite pts\<close> ]) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
326 |
show "connected (S - {p} - pts)" using connected by (metis Diff_insert2) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
327 |
show "open (S - {p})" using \<open>open S\<close> by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
328 |
show " pts \<subseteq> S - {p}" using \<open>insert p pts \<subseteq> S\<close> \<open> p \<notin> pts\<close> by blast |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
329 |
show "f holomorphic_on S - {p} - pts" using holo \<open>p \<notin> pts\<close> by (metis Diff_insert2) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
330 |
show "valid_path g'" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
331 |
unfolding g'_def cp_def using n_circ valid pg g_loop |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
332 |
by (auto intro!:valid_path_join) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
333 |
show "pathfinish g' = pathstart g'" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
334 |
unfolding g'_def cp_def using pg(2) by simp |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
335 |
show "path_image g' \<subseteq> S - {p} - pts" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
336 |
proof - |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
337 |
define s' where "s' \<equiv> S - {p} - pts" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
338 |
have s':"s' = S-insert p pts " unfolding s'_def by auto |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
339 |
then show ?thesis using path_img pg(4) cp(4) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
340 |
by (simp add: g'_def s'_def subset_path_image_join) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
341 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
342 |
note path_join_imp[simp] |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
343 |
show "\<forall>z. z \<notin> S - {p} \<longrightarrow> winding_number g' z = 0" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
344 |
proof clarify |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
345 |
fix z assume z:"z\<notin>S - {p}" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
346 |
have z_notin_cp: "z \<notin> path_image cp" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
347 |
using cp(6) cp_def n_circ(6) z by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
348 |
have z_notin_pg: "z \<notin> path_image pg" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
349 |
by (metis Diff_iff Diff_insert2 pg(4) subsetD z) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
350 |
have "winding_number (g +++ pg +++ cp +++ reversepath pg) z = winding_number g z |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
351 |
+ winding_number (pg +++ cp +++ (reversepath pg)) z" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
352 |
proof (rule winding_number_join) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
353 |
show "path g" using \<open>valid_path g\<close> by (simp add: valid_path_imp_path) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
354 |
show "z \<notin> path_image g" using z path_img by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
355 |
show "path (pg +++ cp +++ reversepath pg)" using pg(3) cp |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
356 |
by (simp add: valid_path_imp_path) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
357 |
next |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
358 |
have "path_image (pg +++ cp +++ reversepath pg) \<subseteq> S - insert p pts" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
359 |
using pg(4) cp(4) by (auto simp:subset_path_image_join) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
360 |
then show "z \<notin> path_image (pg +++ cp +++ reversepath pg)" using z by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
361 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
362 |
show "pathfinish g = pathstart (pg +++ cp +++ reversepath pg)" using g_loop by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
363 |
qed |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
364 |
also have "\<dots> = winding_number g z + (winding_number pg z |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
365 |
+ winding_number (cp +++ (reversepath pg)) z)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
366 |
proof (subst add_left_cancel,rule winding_number_join) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
367 |
show "path pg" and "path (cp +++ reversepath pg)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
368 |
and "pathfinish pg = pathstart (cp +++ reversepath pg)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
369 |
by (auto simp add: valid_path_imp_path) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
370 |
show "z \<notin> path_image pg" using pg(4) z by blast |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
371 |
show "z \<notin> path_image (cp +++ reversepath pg)" using z |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
372 |
by (metis Diff_iff \<open>z \<notin> path_image pg\<close> contra_subsetD cp(4) insertI1 |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
373 |
not_in_path_image_join path_image_reversepath singletonD) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
374 |
qed |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
375 |
also have "\<dots> = winding_number g z + (winding_number pg z |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
376 |
+ (winding_number cp z + winding_number (reversepath pg) z))" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
377 |
by (simp add: valid_path_imp_path winding_number_join z_notin_cp z_notin_pg) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
378 |
also have "\<dots> = winding_number g z + winding_number cp z" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
379 |
by (simp add: valid_path_imp_path winding_number_reversepath z_notin_pg) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
380 |
finally have "winding_number g' z = winding_number g z + winding_number cp z" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
381 |
unfolding g'_def . |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
382 |
moreover have "winding_number g z + winding_number cp z = 0" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
383 |
using winding z \<open>n=winding_number g p\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
384 |
ultimately show "winding_number g' z = 0" unfolding g'_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
385 |
qed |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
386 |
show "\<forall>pa \<in> S - {p}. 0 < h pa \<and> (\<forall>w\<in>cball pa (h pa). w \<in> S - {p} \<and> (w \<noteq> pa \<longrightarrow> w \<notin> pts))" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
387 |
using h by fastforce |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
388 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
389 |
moreover have "contour_integral g' f = contour_integral g f |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
390 |
- winding_number g p * contour_integral p_circ f" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
391 |
proof - |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
392 |
have *: "f contour_integrable_on g" "f contour_integrable_on pg" "f contour_integrable_on cp" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
393 |
by (auto simp add: open_Diff[OF \<open>open S\<close>,OF finite_imp_closed[OF fin]] |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
394 |
intro!: contour_integrable_holomorphic_simple[OF holo _ _ path_img]) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
395 |
have "contour_integral g' f = contour_integral g f + contour_integral pg f |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
396 |
+ contour_integral cp f + contour_integral (reversepath pg) f" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
397 |
using * by (simp add: g'_def contour_integrable_reversepath_eq) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
398 |
also have "\<dots> = contour_integral g f + contour_integral cp f" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
399 |
using contour_integral_reversepath |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
400 |
by (auto simp add:contour_integrable_reversepath) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
401 |
also have "\<dots> = contour_integral g f - winding_number g p * contour_integral p_circ f" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
402 |
using \<open>n=winding_number g p\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
403 |
finally show ?thesis . |
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 "winding_number g' p' = winding_number g p'" when "p'\<in>pts" for p' |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
406 |
proof - |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
407 |
obtain [simp]: "p' \<notin> path_image g" "p' \<notin> path_image pg" "p'\<notin>path_image cp" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
408 |
using "2.prems"(8) that by (metis Diff_iff Diff_insert2 \<open>p' \<in> pts\<close> cp(4) pg(4) subsetD) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
409 |
have "winding_number g' p' = winding_number g p' + winding_number pg p' |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
410 |
+ winding_number (cp +++ reversepath pg) p'" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
411 |
by (simp add: g'_def not_in_path_image_join valid_path_imp_path winding_number_join) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
412 |
also have "\<dots> = winding_number g p'" using that |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
413 |
by (simp add: valid_path_imp_path winding_number_join winding_number_reversepath) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
414 |
finally show ?thesis . |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
415 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
416 |
ultimately show ?case unfolding p_circ_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
417 |
apply (subst (asm) sum.cong[OF refl, |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
418 |
of pts _ "\<lambda>p. winding_number g p * contour_integral (circlepath p (h p)) f"]) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
419 |
by (auto simp: sum.insert[OF \<open>finite pts\<close> \<open>p\<notin>pts\<close>] algebra_simps) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
420 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
421 |
|
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
422 |
lemma Cauchy_theorem_singularities: |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
423 |
assumes "open S" "connected S" "finite pts" and |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
424 |
holo: "f holomorphic_on S-pts" and |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
425 |
"valid_path g" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
426 |
loop:"pathfinish g = pathstart g" and |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
427 |
"path_image g \<subseteq> S-pts" and |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
428 |
homo:"\<forall>z. (z \<notin> S) \<longrightarrow> winding_number g z = 0" and |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
429 |
avoid:"\<forall>p\<in>S. h p>0 \<and> (\<forall>w\<in>cball p (h p). w\<in>S \<and> (w\<noteq>p \<longrightarrow> w \<notin> pts))" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
430 |
shows "contour_integral g f = (\<Sum>p\<in>pts. winding_number g p * contour_integral (circlepath p (h p)) f)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
431 |
(is "?L=?R") |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
432 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
433 |
define circ where "circ \<equiv> \<lambda>p. winding_number g p * contour_integral (circlepath p (h p)) f" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
434 |
define pts1 where "pts1 \<equiv> pts \<inter> S" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
435 |
define pts2 where "pts2 \<equiv> pts - pts1" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
436 |
have "pts=pts1 \<union> pts2" "pts1 \<inter> pts2 = {}" "pts2 \<inter> S={}" "pts1\<subseteq>S" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
437 |
unfolding pts1_def pts2_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
438 |
have "contour_integral g f = (\<Sum>p\<in>pts1. circ p)" unfolding circ_def |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
439 |
proof (rule Cauchy_theorem_aux[OF \<open>open S\<close> _ _ \<open>pts1\<subseteq>S\<close> _ \<open>valid_path g\<close> loop _ homo]) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
440 |
have "finite pts1" unfolding pts1_def using \<open>finite pts\<close> by auto |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
441 |
then show "connected (S - pts1)" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
442 |
using \<open>open S\<close> \<open>connected S\<close> connected_open_delete_finite[of S] by auto |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
443 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
444 |
show "finite pts1" using \<open>pts = pts1 \<union> pts2\<close> assms(3) by auto |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
445 |
show "f holomorphic_on S - pts1" by (metis Diff_Int2 Int_absorb holo pts1_def) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
446 |
show "path_image g \<subseteq> S - pts1" using assms(7) pts1_def by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
447 |
show "\<forall>p\<in>S. 0 < h p \<and> (\<forall>w\<in>cball p (h p). w \<in> S \<and> (w \<noteq> p \<longrightarrow> w \<notin> pts1))" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
448 |
by (simp add: avoid pts1_def) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
449 |
qed |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
450 |
moreover have "sum circ pts2 = 0" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
451 |
by (metis \<open>pts2 \<inter> S = {}\<close> circ_def disjoint_iff_not_equal homo mult_zero_left sum.neutral) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
452 |
moreover have "?R=sum circ pts1 + sum circ pts2" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
453 |
unfolding circ_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
454 |
using sum.union_disjoint[OF _ _ \<open>pts1 \<inter> pts2 = {}\<close>] \<open>finite pts\<close> \<open>pts=pts1 \<union> pts2\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
455 |
by blast |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
456 |
ultimately show ?thesis |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
457 |
by simp |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
458 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
459 |
|
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
460 |
theorem Residue_theorem: |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
461 |
fixes S pts::"complex set" and f::"complex \<Rightarrow> complex" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
462 |
and g::"real \<Rightarrow> complex" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
463 |
assumes "open S" "connected S" "finite pts" and |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
464 |
holo:"f holomorphic_on S-pts" and |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
465 |
"valid_path g" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
466 |
loop:"pathfinish g = pathstart g" and |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
467 |
"path_image g \<subseteq> S-pts" and |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
468 |
homo:"\<forall>z. (z \<notin> S) \<longrightarrow> winding_number g z = 0" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
469 |
shows "contour_integral g f = 2 * pi * \<i> *(\<Sum>p\<in>pts. winding_number g p * residue f p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
470 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
471 |
define c where "c \<equiv> 2 * pi * \<i>" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
472 |
obtain h where avoid:"\<forall>p\<in>S. h p>0 \<and> (\<forall>w\<in>cball p (h p). w\<in>S \<and> (w\<noteq>p \<longrightarrow> w \<notin> pts))" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
473 |
using finite_cball_avoid[OF \<open>open S\<close> \<open>finite pts\<close>] by metis |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
474 |
have "contour_integral g f |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
475 |
= (\<Sum>p\<in>pts. winding_number g p * contour_integral (circlepath p (h p)) f)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
476 |
using Cauchy_theorem_singularities[OF assms avoid] . |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
477 |
also have "\<dots> = (\<Sum>p\<in>pts. c * winding_number g p * residue f p)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
478 |
proof (intro sum.cong) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
479 |
show "pts = pts" by simp |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
480 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
481 |
fix x assume "x \<in> pts" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
482 |
show "winding_number g x * contour_integral (circlepath x (h x)) f |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
483 |
= c * winding_number g x * residue f x" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
484 |
proof (cases "x\<in>S") |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
485 |
case False |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
486 |
then have "winding_number g x=0" using homo by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
487 |
thus ?thesis by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
488 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
489 |
case True |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
490 |
have "contour_integral (circlepath x (h x)) f = c* residue f x" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
491 |
using \<open>x\<in>pts\<close> \<open>finite pts\<close> avoid[rule_format, OF True] |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
492 |
apply (intro base_residue[of "S-(pts-{x})",THEN contour_integral_unique,folded c_def]) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
493 |
by (auto intro:holomorphic_on_subset[OF holo] open_Diff[OF \<open>open S\<close> finite_imp_closed]) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
494 |
then show ?thesis by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
495 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
496 |
qed |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
497 |
also have "\<dots> = c * (\<Sum>p\<in>pts. winding_number g p * residue f p)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
498 |
by (simp add: sum_distrib_left algebra_simps) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
499 |
finally show ?thesis unfolding c_def . |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
500 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
501 |
|
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
502 |
subsection \<open>The argument principle\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
503 |
|
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
504 |
theorem argument_principle: |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
505 |
fixes f::"complex \<Rightarrow> complex" and poles S:: "complex set" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
506 |
defines "pz \<equiv> {w\<in>S. f w = 0 \<or> w \<in> poles}" \<comment> \<open>\<^term>\<open>pz\<close> is the set of poles and zeros\<close> |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
507 |
assumes "open S" "connected S" and |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
508 |
f_holo:"f holomorphic_on S-poles" and |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
509 |
h_holo:"h holomorphic_on S" and |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
510 |
"valid_path g" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
511 |
loop:"pathfinish g = pathstart g" and |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
512 |
path_img:"path_image g \<subseteq> S - pz" and |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
513 |
homo:"\<forall>z. (z \<notin> S) \<longrightarrow> winding_number g z = 0" and |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
514 |
finite:"finite pz" and |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
515 |
poles:"\<forall>p\<in>S\<inter>poles. is_pole f p" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
516 |
shows "contour_integral g (\<lambda>x. deriv f x * h x / f x) = 2 * pi * \<i> * |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
517 |
(\<Sum>p\<in>pz. winding_number g p * h p * zorder f p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
518 |
(is "?L=?R") |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
519 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
520 |
define c where "c \<equiv> 2 * complex_of_real pi * \<i> " |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
521 |
define ff where "ff \<equiv> (\<lambda>x. deriv f x * h x / f x)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
522 |
define cont where "cont \<equiv> \<lambda>ff p e. (ff has_contour_integral c * zorder f p * h p ) (circlepath p e)" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
523 |
define avoid where "avoid \<equiv> \<lambda>p e. \<forall>w\<in>cball p e. w \<in> S \<and> (w \<noteq> p \<longrightarrow> w \<notin> pz)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
524 |
|
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
525 |
have "\<exists>e>0. avoid p e \<and> (p\<in>pz \<longrightarrow> cont ff p e)" when "p\<in>S" for p |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
526 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
527 |
obtain e1 where "e1>0" and e1_avoid:"avoid p e1" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
528 |
using finite_cball_avoid[OF \<open>open S\<close> finite] \<open>p\<in>S\<close> unfolding avoid_def by auto |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
529 |
have "\<exists>e2>0. cball p e2 \<subseteq> ball p e1 \<and> cont ff p e2" when "p\<in>pz" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
530 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
531 |
define po where "po \<equiv> zorder f p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
532 |
define pp where "pp \<equiv> zor_poly f p" |
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
|
533 |
define f' where "f' \<equiv> \<lambda>w. pp w * (w - p) powi po" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
534 |
define ff' where "ff' \<equiv> (\<lambda>x. deriv f' x * h x / f' x)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
535 |
obtain r where "pp p\<noteq>0" "r>0" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
536 |
"r<e1" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
537 |
pp_holo:"pp holomorphic_on cball p r" and |
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
|
538 |
pp_po:"(\<forall>w\<in>cball p r-{p}. f w = pp w * (w - p) powi po \<and> pp w \<noteq> 0)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
539 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
540 |
have "isolated_singularity_at f p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
541 |
proof - |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
542 |
have "ball p e1 - {p} \<subseteq> S - poles" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
543 |
using avoid_def e1_avoid pz_def by fastforce |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
544 |
then have "f holomorphic_on ball p e1 - {p}" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
545 |
by (intro holomorphic_on_subset[OF f_holo]) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
546 |
then show ?thesis unfolding isolated_singularity_at_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
547 |
using \<open>e1>0\<close> analytic_on_open open_delete by blast |
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 |
moreover have "not_essential f p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
550 |
proof (cases "is_pole f p") |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
551 |
case True |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
552 |
then show ?thesis unfolding not_essential_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
553 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
554 |
case False |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
555 |
then have "p\<in>S-poles" using \<open>p\<in>S\<close> poles unfolding pz_def by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
556 |
moreover have "open (S-poles)" |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
557 |
proof - |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
558 |
have "closed (S \<inter> poles)" |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
559 |
using finite by (simp add: pz_def finite_imp_closed rev_finite_subset subset_eq) |
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
560 |
then show ?thesis |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
561 |
by (metis Diff_Compl Diff_Diff_Int Diff_eq \<open>open S\<close> open_Diff) |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
562 |
qed |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
563 |
ultimately have "isCont f p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
564 |
using holomorphic_on_imp_continuous_on[OF f_holo] continuous_on_eq_continuous_at |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
565 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
566 |
then show ?thesis unfolding isCont_def not_essential_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
567 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
568 |
moreover have "\<exists>\<^sub>F w in at p. f w \<noteq> 0 " |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
569 |
proof (rule ccontr) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
570 |
assume "\<not> (\<exists>\<^sub>F w in at p. f w \<noteq> 0)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
571 |
then have "\<forall>\<^sub>F w in at p. f w= 0" unfolding frequently_def by auto |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
572 |
then obtain r1 where "r1>0" and r1:"\<forall>w\<in>ball p r1 - {p}. f w =0" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
573 |
unfolding eventually_at by (auto simp add:dist_commute) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
574 |
obtain r2 where "r2>0" and r2: "ball p r2 \<subseteq> S" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
575 |
using \<open>p\<in>S\<close> \<open>open S\<close> openE by blast |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
576 |
define rr where "rr=min r1 r2" |
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
577 |
|
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
578 |
from r1 r2 |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
579 |
have "ball p rr - {p} \<subseteq> {w\<in> S \<inter> ball p rr-{p}. f w=0}" |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
580 |
unfolding rr_def by auto |
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
581 |
moreover have "infinite (ball p rr - {p})" |
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
582 |
using \<open>r1>0\<close> \<open>r2>0\<close> finite_imp_not_open |
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
583 |
unfolding rr_def by fastforce |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
584 |
ultimately have "infinite {w\<in>S \<inter> ball p rr-{p}. f w=0}" using infinite_super by blast |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
585 |
then have "infinite pz" |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
586 |
unfolding pz_def by (smt (verit) infinite_super Collect_mono_iff DiffE Int_iff) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
587 |
then show False using \<open>finite pz\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
588 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
589 |
ultimately obtain r where "pp p \<noteq> 0" and r:"r>0" "pp holomorphic_on cball p 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
|
590 |
"(\<forall>w\<in>cball p r - {p}. f w = pp w * (w - p) powi po \<and> pp w \<noteq> 0)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
591 |
using zorder_exist[of f p,folded po_def pp_def] by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
592 |
define r1 where "r1=min r e1 / 2" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
593 |
have "r1<e1" unfolding r1_def using \<open>e1>0\<close> \<open>r>0\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
594 |
moreover have "r1>0" "pp holomorphic_on cball p r1" |
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
|
595 |
"(\<forall>w\<in>cball p r1 - {p}. f w = pp w * (w - p) powi po \<and> pp w \<noteq> 0)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
596 |
unfolding r1_def using \<open>e1>0\<close> r by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
597 |
ultimately show ?thesis using that \<open>pp p\<noteq>0\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
598 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
599 |
|
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
600 |
define e2 where "e2 \<equiv> r/2" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
601 |
have "e2>0" using \<open>r>0\<close> unfolding e2_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
602 |
define anal where "anal \<equiv> \<lambda>w. deriv pp w * h w / pp w" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
603 |
define prin where "prin \<equiv> \<lambda>w. po * h w / (w - p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
604 |
have "((\<lambda>w. prin w + anal w) has_contour_integral c * po * h p) (circlepath p e2)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
605 |
proof (rule has_contour_integral_add[of _ _ _ _ 0,simplified]) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
606 |
have "ball p r \<subseteq> S" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
607 |
using \<open>r<e1\<close> avoid_def ball_subset_cball e1_avoid by (simp add: subset_eq) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
608 |
then have "cball p e2 \<subseteq> S" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
609 |
using \<open>r>0\<close> unfolding e2_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
610 |
then have "(\<lambda>w. po * h w) holomorphic_on cball p e2" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
611 |
using h_holo by (auto intro!: holomorphic_intros) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
612 |
then show "(prin has_contour_integral c * po * h p ) (circlepath p e2)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
613 |
using Cauchy_integral_circlepath_simple[folded c_def, of "\<lambda>w. po * h w"] \<open>e2>0\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
614 |
unfolding prin_def by (auto simp add: mult.assoc) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
615 |
have "anal holomorphic_on ball p r" unfolding anal_def |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
616 |
using pp_holo h_holo pp_po \<open>ball p r \<subseteq> S\<close> \<open>pp p\<noteq>0\<close> |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
617 |
by (auto intro!: holomorphic_intros) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
618 |
then show "(anal has_contour_integral 0) (circlepath p e2)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
619 |
using e2_def \<open>r>0\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
620 |
by (auto elim!: Cauchy_theorem_disc_simple) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
621 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
622 |
then have "cont ff' p e2" unfolding cont_def po_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
623 |
proof (elim has_contour_integral_eq) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
624 |
fix w assume "w \<in> path_image (circlepath p e2)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
625 |
then have "w\<in>ball p r" and "w\<noteq>p" unfolding e2_def using \<open>r>0\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
626 |
define wp where "wp \<equiv> w-p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
627 |
have "wp\<noteq>0" and "pp w \<noteq>0" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
628 |
unfolding wp_def using \<open>w\<noteq>p\<close> \<open>w\<in>ball p r\<close> pp_po 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
|
629 |
moreover have der_f':"deriv f' w = po * pp w * (w-p) powi (po - 1) + deriv pp w * (w-p) powi po" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
630 |
proof (rule DERIV_imp_deriv) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
631 |
have "(pp has_field_derivative (deriv pp w)) (at w)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
632 |
using DERIV_deriv_iff_has_field_derivative pp_holo \<open>w\<noteq>p\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
633 |
by (meson open_ball \<open>w \<in> ball p r\<close> ball_subset_cball holomorphic_derivI holomorphic_on_subset) |
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
|
634 |
then show " (f' has_field_derivative of_int po * pp w * (w - p) powi (po - 1) |
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
|
635 |
+ deriv pp w * (w - p) powi po) (at w)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
636 |
unfolding f'_def using \<open>w\<noteq>p\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
637 |
by (auto intro!: derivative_eq_intros DERIV_cong[OF has_field_derivative_powr_of_int]) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
638 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
639 |
ultimately show "prin w + anal w = ff' w" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
640 |
unfolding f'_def ff'_def prin_def anal_def |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
641 |
apply (simp add: field_simps flip: wp_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
|
642 |
by (metis (no_types, lifting) mult.commute power_int_minus_mult) |
71201
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 |
then have "cont ff p e2" unfolding cont_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
645 |
proof (elim has_contour_integral_eq) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
646 |
fix w assume "w \<in> path_image (circlepath p e2)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
647 |
then have "w\<in>ball p r" and "w\<noteq>p" unfolding e2_def using \<open>r>0\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
648 |
have "deriv f' w = deriv f w" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
649 |
proof (rule complex_derivative_transform_within_open[where s="ball p r - {p}"]) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
650 |
show "f' holomorphic_on ball p r - {p}" unfolding f'_def using pp_holo |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
651 |
by (auto intro!: holomorphic_intros) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
652 |
next |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
653 |
have "ball p e1 - {p} \<subseteq> S - poles" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
654 |
using ball_subset_cball e1_avoid[unfolded avoid_def] unfolding pz_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
655 |
by auto |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
656 |
then have "ball p r - {p} \<subseteq> S - poles" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
657 |
using \<open>r<e1\<close> by force |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
658 |
then show "f holomorphic_on ball p r - {p}" using f_holo |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
659 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
660 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
661 |
show "open (ball p r - {p})" by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
662 |
show "w \<in> ball p r - {p}" using \<open>w\<in>ball p r\<close> \<open>w\<noteq>p\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
663 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
664 |
fix x assume "x \<in> ball p r - {p}" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
665 |
then show "f' x = f x" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
666 |
using pp_po unfolding f'_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
667 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
668 |
moreover have " f' w = f w " |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
669 |
using \<open>w \<in> ball p r\<close> ball_subset_cball subset_iff pp_po \<open>w\<noteq>p\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
670 |
unfolding f'_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
671 |
ultimately show "ff' w = ff w" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
672 |
unfolding ff'_def ff_def by simp |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
673 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
674 |
moreover have "cball p e2 \<subseteq> ball p e1" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
675 |
using \<open>0 < r\<close> \<open>r<e1\<close> e2_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
676 |
ultimately show ?thesis using \<open>e2>0\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
677 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
678 |
then obtain e2 where e2:"p\<in>pz \<longrightarrow> e2>0 \<and> cball p e2 \<subseteq> ball p e1 \<and> cont ff p e2" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
679 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
680 |
define e4 where "e4 \<equiv> if p\<in>pz then e2 else e1" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
681 |
have "e4>0" using e2 \<open>e1>0\<close> unfolding e4_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
682 |
moreover have "avoid p e4" using e2 \<open>e1>0\<close> e1_avoid unfolding e4_def avoid_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
683 |
moreover have "p\<in>pz \<longrightarrow> cont ff p e4" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
684 |
by (auto simp add: e2 e4_def) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
685 |
ultimately show ?thesis by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
686 |
qed |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
687 |
then obtain get_e where get_e:"\<forall>p\<in>S. get_e p>0 \<and> avoid p (get_e p) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
688 |
\<and> (p\<in>pz \<longrightarrow> cont ff p (get_e p))" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
689 |
by metis |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
690 |
define ci where "ci \<equiv> \<lambda>p. contour_integral (circlepath p (get_e p)) ff" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
691 |
define w where "w \<equiv> \<lambda>p. winding_number g p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
692 |
have "contour_integral g ff = (\<Sum>p\<in>pz. w p * ci p)" unfolding ci_def w_def |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
693 |
proof (rule Cauchy_theorem_singularities[OF \<open>open S\<close> \<open>connected S\<close> finite _ \<open>valid_path g\<close> loop |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
694 |
path_img homo]) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
695 |
have "open (S - pz)" using open_Diff[OF _ finite_imp_closed[OF finite]] \<open>open S\<close> by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
696 |
then show "ff holomorphic_on S - pz" unfolding ff_def using f_holo h_holo |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
697 |
by (auto intro!: holomorphic_intros simp add:pz_def) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
698 |
next |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
699 |
show "\<forall>p\<in>S. 0 < get_e p \<and> (\<forall>w\<in>cball p (get_e p). w \<in> S \<and> (w \<noteq> p \<longrightarrow> w \<notin> pz))" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
700 |
using get_e using avoid_def by blast |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
701 |
qed |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
702 |
also have "\<dots> = (\<Sum>p\<in>pz. c * w p * h p * zorder f p)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
703 |
proof (rule sum.cong[of pz pz,simplified]) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
704 |
fix p assume "p \<in> pz" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
705 |
show "w p * ci p = c * w p * h p * (zorder f p)" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
706 |
proof (cases "p\<in>S") |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
707 |
assume "p \<in> S" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
708 |
have "ci p = c * h p * (zorder f p)" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
709 |
unfolding ci_def |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
710 |
using \<open>p \<in> S\<close> \<open>p \<in> pz\<close> cont_def contour_integral_unique get_e by fastforce |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
711 |
thus ?thesis by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
712 |
next |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
713 |
assume "p\<notin>S" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
714 |
then have "w p=0" using homo unfolding w_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
715 |
then show ?thesis by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
716 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
717 |
qed |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
718 |
also have "\<dots> = c*(\<Sum>p\<in>pz. w p * h p * zorder f p)" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
719 |
unfolding sum_distrib_left by (simp add:algebra_simps) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
720 |
finally have "contour_integral g ff = c * (\<Sum>p\<in>pz. w p * h p * of_int (zorder f p))" . |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
721 |
then show ?thesis unfolding ff_def c_def w_def by simp |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
722 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
723 |
|
73048
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
724 |
|
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
725 |
subsection \<open>Coefficient asymptotics for generating functions\<close> |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
726 |
|
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
727 |
text \<open> |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
728 |
For a formal power series that has a meromorphic continuation on some disc in the |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
729 |
context plane, we can use the Residue Theorem to extract precise asymptotic information |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
730 |
from the residues at the poles. This can be used to derive the asymptotic behaviour |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
731 |
of the coefficients (\<open>a\<^sub>n \<sim> \<dots>\<close>). If the function is meromorphic on the entire |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
732 |
complex plane, one can even derive a full asymptotic expansion. |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
733 |
|
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
734 |
We will first show the relationship between the coefficients and the sum over the residues |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
735 |
with an explicit remainder term (the contour integral along the circle used in the |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
736 |
Residue theorem). |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
737 |
\<close> |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
738 |
theorem |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
739 |
fixes f :: "complex \<Rightarrow> complex" and n :: nat and r :: real |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
740 |
defines "g \<equiv> (\<lambda>w. f w / w ^ Suc n)" and "\<gamma> \<equiv> circlepath 0 r" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
741 |
assumes "open A" "connected A" "cball 0 r \<subseteq> A" "r > 0" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
742 |
assumes "f holomorphic_on A - S" "S \<subseteq> ball 0 r" "finite S" "0 \<notin> S" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
743 |
shows fps_coeff_conv_residues: |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
744 |
"(deriv ^^ n) f 0 / fact n = |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
745 |
contour_integral \<gamma> g / (2 * pi * \<i>) - (\<Sum>z\<in>S. residue g z)" (is ?thesis1) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
746 |
and fps_coeff_residues_bound: |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
747 |
"(\<And>z. norm z = r \<Longrightarrow> z \<notin> k \<Longrightarrow> norm (f z) \<le> C) \<Longrightarrow> C \<ge> 0 \<Longrightarrow> finite k \<Longrightarrow> |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
748 |
norm ((deriv ^^ n) f 0 / fact n + (\<Sum>z\<in>S. residue g z)) \<le> C / r ^ n" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
749 |
proof - |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
750 |
have holo: "g holomorphic_on A - insert 0 S" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
751 |
unfolding g_def using assms by (auto intro!: holomorphic_intros) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
752 |
have "contour_integral \<gamma> g = 2 * pi * \<i> * (\<Sum>z\<in>insert 0 S. winding_number \<gamma> z * residue g z)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
753 |
proof (rule Residue_theorem) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
754 |
show "g holomorphic_on A - insert 0 S" by fact |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
755 |
from assms show "\<forall>z. z \<notin> A \<longrightarrow> winding_number \<gamma> z = 0" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
756 |
unfolding \<gamma>_def by (intro allI impI winding_number_zero_outside[of _ "cball 0 r"]) auto |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
757 |
qed (insert assms, auto simp: \<gamma>_def) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
758 |
also have "winding_number \<gamma> z = 1" if "z \<in> insert 0 S" for z |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
759 |
unfolding \<gamma>_def using assms that by (intro winding_number_circlepath) auto |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
760 |
hence "(\<Sum>z\<in>insert 0 S. winding_number \<gamma> z * residue g z) = (\<Sum>z\<in>insert 0 S. residue g z)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
761 |
by (intro sum.cong) simp_all |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
762 |
also have "\<dots> = residue g 0 + (\<Sum>z\<in>S. residue g z)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
763 |
using \<open>0 \<notin> S\<close> and \<open>finite S\<close> by (subst sum.insert) auto |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
764 |
also from \<open>r > 0\<close> have "0 \<in> cball 0 r" by simp |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
765 |
with assms have "0 \<in> A - S" by blast |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
766 |
with assms have "residue g 0 = (deriv ^^ n) f 0 / fact n" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
767 |
unfolding g_def by (subst residue_holomorphic_over_power'[of "A - S"]) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
768 |
(auto simp: finite_imp_closed) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
769 |
finally show ?thesis1 |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
770 |
by (simp add: field_simps) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
771 |
|
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
772 |
assume C: "\<And>z. norm z = r \<Longrightarrow> z \<notin> k \<Longrightarrow> norm (f z) \<le> C" "C \<ge> 0" and k: "finite k" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
773 |
have "(deriv ^^ n) f 0 / fact n + (\<Sum>z\<in>S. residue g z) = contour_integral \<gamma> g / (2 * pi * \<i>)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
774 |
using \<open>?thesis1\<close> by (simp add: algebra_simps) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
775 |
also have "norm \<dots> = norm (contour_integral \<gamma> g) / (2 * pi)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
776 |
by (simp add: norm_divide norm_mult) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
777 |
also have "norm (contour_integral \<gamma> g) \<le> C / r ^ Suc n * (2 * pi * r)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
778 |
proof (rule has_contour_integral_bound_circlepath_strong) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
779 |
from \<open>open A\<close> and \<open>finite S\<close> have "open (A - insert 0 S)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
780 |
by (blast intro: finite_imp_closed) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
781 |
with assms show "(g has_contour_integral contour_integral \<gamma> g) (circlepath 0 r)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
782 |
unfolding \<gamma>_def |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
783 |
by (intro has_contour_integral_integral contour_integrable_holomorphic_simple [OF holo]) auto |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
784 |
next |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
785 |
fix z assume z: "norm (z - 0) = r" "z \<notin> k" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
786 |
hence "norm (g z) = norm (f z) / r ^ Suc n" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
787 |
by (simp add: norm_divide g_def norm_mult norm_power) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
788 |
also have "\<dots> \<le> C / r ^ Suc n" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
789 |
using k and \<open>r > 0\<close> and z by (intro divide_right_mono C zero_le_power) auto |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
790 |
finally show "norm (g z) \<le> C / r ^ Suc n" . |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
791 |
qed (insert C(2) k \<open>r > 0\<close>, auto) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
792 |
also from \<open>r > 0\<close> have "C / r ^ Suc n * (2 * pi * r) / (2 * pi) = C / r ^ n" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
793 |
by simp |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
794 |
finally show "norm ((deriv ^^ n) f 0 / fact n + (\<Sum>z\<in>S. residue g z)) \<le> \<dots>" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
795 |
by - (simp_all add: divide_right_mono) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
796 |
qed |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
797 |
|
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
798 |
text \<open> |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
799 |
Since the circle is fixed, we can get an upper bound on the values of the generating |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
800 |
function on the circle and therefore show that the integral is $O(r^{-n})$. |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
801 |
\<close> |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
802 |
corollary fps_coeff_residues_bigo: |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
803 |
fixes f :: "complex \<Rightarrow> complex" and r :: real |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
804 |
assumes "open A" "connected A" "cball 0 r \<subseteq> A" "r > 0" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
805 |
assumes "f holomorphic_on A - S" "S \<subseteq> ball 0 r" "finite S" "0 \<notin> S" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
806 |
assumes g: "eventually (\<lambda>n. g n = -(\<Sum>z\<in>S. residue (\<lambda>z. f z / z ^ Suc n) z)) sequentially" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
807 |
(is "eventually (\<lambda>n. _ = -?g' n) _") |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
808 |
shows "(\<lambda>n. (deriv ^^ n) f 0 / fact n - g n) \<in> O(\<lambda>n. 1 / r ^ n)" (is "(\<lambda>n. ?c n - _) \<in> O(_)") |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
809 |
proof - |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
810 |
from assms have "compact (f ` sphere 0 r)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
811 |
by (intro compact_continuous_image holomorphic_on_imp_continuous_on |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
812 |
holomorphic_on_subset[OF \<open>f holomorphic_on A - S\<close>]) auto |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
813 |
hence "bounded (f ` sphere 0 r)" by (rule compact_imp_bounded) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
814 |
then obtain C where C: "\<And>z. z \<in> sphere 0 r \<Longrightarrow> norm (f z) \<le> C" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
815 |
by (auto simp: bounded_iff sphere_def) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
816 |
have "0 \<le> norm (f (of_real r))" by simp |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
817 |
also from C[of "of_real r"] and \<open>r > 0\<close> have "\<dots> \<le> C" by simp |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
818 |
finally have C_nonneg: "C \<ge> 0" . |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
819 |
|
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
820 |
have "(\<lambda>n. ?c n + ?g' n) \<in> O(\<lambda>n. of_real (1 / r ^ n))" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
821 |
proof (intro bigoI[of _ C] always_eventually allI ) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
822 |
fix n :: nat |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
823 |
from assms and C and C_nonneg have "norm (?c n + ?g' n) \<le> C / r ^ n" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
824 |
by (intro fps_coeff_residues_bound[where A = A and k = "{}"]) auto |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
825 |
also have "\<dots> = C * norm (complex_of_real (1 / r ^ n))" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
826 |
using \<open>r > 0\<close> by (simp add: norm_divide norm_power) |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
827 |
finally show "norm (?c n + ?g' n) \<le> \<dots>" . |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
828 |
qed |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
829 |
also have "?this \<longleftrightarrow> (\<lambda>n. ?c n - g n) \<in> O(\<lambda>n. of_real (1 / r ^ n))" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
830 |
by (intro landau_o.big.in_cong eventually_mono[OF g]) simp_all |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
831 |
finally show ?thesis . |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
832 |
qed |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
833 |
|
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
834 |
corollary fps_coeff_residues_bigo': |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
835 |
fixes f :: "complex \<Rightarrow> complex" and r :: real |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
836 |
assumes exp: "f has_fps_expansion F" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
837 |
assumes "open A" "connected A" "cball 0 r \<subseteq> A" "r > 0" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
838 |
assumes "f holomorphic_on A - S" "S \<subseteq> ball 0 r" "finite S" "0 \<notin> S" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
839 |
assumes "eventually (\<lambda>n. g n = -(\<Sum>z\<in>S. residue (\<lambda>z. f z / z ^ Suc n) z)) sequentially" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
840 |
(is "eventually (\<lambda>n. _ = -?g' n) _") |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
841 |
shows "(\<lambda>n. fps_nth F n - g n) \<in> O(\<lambda>n. 1 / r ^ n)" (is "(\<lambda>n. ?c n - _) \<in> O(_)") |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
842 |
proof - |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
843 |
have "fps_nth F = (\<lambda>n. (deriv ^^ n) f 0 / fact n)" |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
844 |
using fps_nth_fps_expansion[OF exp] by (intro ext) simp_all |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
845 |
with fps_coeff_residues_bigo[OF assms(2-)] show ?thesis by simp |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
846 |
qed |
7ad9f197ca7e
HOL-Complex_Analysis: coefficient asymptotics for meromorphic functions
Manuel Eberl <eberlm@in.tum.de>
parents:
71201
diff
changeset
|
847 |
|
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
848 |
subsection \<open>Rouche's theorem \<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
849 |
|
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
850 |
theorem Rouche_theorem: |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
851 |
fixes f g::"complex \<Rightarrow> complex" and s:: "complex set" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
852 |
defines "fg\<equiv>(\<lambda>p. f p + g p)" |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
853 |
defines "zeros_fg\<equiv>{p\<in>s. fg p = 0}" and "zeros_f\<equiv>{p\<in>s. f p = 0}" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
854 |
assumes |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
855 |
"open s" and "connected s" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
856 |
"finite zeros_fg" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
857 |
"finite zeros_f" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
858 |
f_holo:"f holomorphic_on s" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
859 |
g_holo:"g holomorphic_on s" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
860 |
"valid_path \<gamma>" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
861 |
loop:"pathfinish \<gamma> = pathstart \<gamma>" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
862 |
path_img:"path_image \<gamma> \<subseteq> s " and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
863 |
path_less:"\<forall>z\<in>path_image \<gamma>. cmod(f z) > cmod(g z)" and |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
864 |
homo:"\<forall>z. (z \<notin> s) \<longrightarrow> winding_number \<gamma> z = 0" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
865 |
shows "(\<Sum>p\<in>zeros_fg. winding_number \<gamma> p * zorder fg p) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
866 |
= (\<Sum>p\<in>zeros_f. winding_number \<gamma> p * zorder f p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
867 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
868 |
have path_fg:"path_image \<gamma> \<subseteq> s - zeros_fg" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
869 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
870 |
have False when "z\<in>path_image \<gamma>" and "f z + g z=0" for z |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
871 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
872 |
have "cmod (f z) > cmod (g z)" using \<open>z\<in>path_image \<gamma>\<close> path_less by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
873 |
moreover have "f z = - g z" using \<open>f z + g z =0\<close> by (simp add: eq_neg_iff_add_eq_0) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
874 |
then have "cmod (f z) = cmod (g z)" by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
875 |
ultimately show False by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
876 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
877 |
then show ?thesis unfolding zeros_fg_def fg_def using path_img by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
878 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
879 |
have path_f:"path_image \<gamma> \<subseteq> s - zeros_f" |
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 False when "z\<in>path_image \<gamma>" and "f z =0" for z |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
882 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
883 |
have "cmod (g z) < cmod (f z) " using \<open>z\<in>path_image \<gamma>\<close> path_less by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
884 |
then have "cmod (g z) < 0" using \<open>f z=0\<close> by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
885 |
then show False by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
886 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
887 |
then show ?thesis unfolding zeros_f_def using path_img by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
888 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
889 |
define w where "w \<equiv> \<lambda>p. winding_number \<gamma> p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
890 |
define c where "c \<equiv> 2 * complex_of_real pi * \<i>" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
891 |
define h where "h \<equiv> \<lambda>p. g p / f p + 1" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
892 |
obtain spikes |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
893 |
where "finite spikes" and spikes: "\<forall>x\<in>{0..1} - spikes. \<gamma> differentiable at x" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
894 |
using \<open>valid_path \<gamma>\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
895 |
by (auto simp: valid_path_def piecewise_C1_differentiable_on_def C1_differentiable_on_eq) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
896 |
have h_contour:"((\<lambda>x. deriv h x / h x) has_contour_integral 0) \<gamma>" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
897 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
898 |
have outside_img:"0 \<in> outside (path_image (h o \<gamma>))" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
899 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
900 |
have "h p \<in> ball 1 1" when "p\<in>path_image \<gamma>" for p |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
901 |
proof - |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
902 |
have "cmod (g p/f p) <1" |
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
903 |
by (smt (verit) divide_less_eq_1_pos norm_divide norm_ge_zero path_less that) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
904 |
then show ?thesis |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
905 |
unfolding h_def by (auto simp add:dist_complex_def) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
906 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
907 |
then have "path_image (h o \<gamma>) \<subseteq> ball 1 1" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
908 |
by (simp add: image_subset_iff path_image_compose) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
909 |
moreover have " (0::complex) \<notin> ball 1 1" by (simp add: dist_norm) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
910 |
ultimately show "?thesis" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
911 |
using convex_in_outside[of "ball 1 1" 0] outside_mono by blast |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
912 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
913 |
have valid_h:"valid_path (h \<circ> \<gamma>)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
914 |
proof (rule valid_path_compose_holomorphic[OF \<open>valid_path \<gamma>\<close> _ _ path_f]) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
915 |
show "h holomorphic_on s - zeros_f" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
916 |
unfolding h_def using f_holo g_holo |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
917 |
by (auto intro!: holomorphic_intros simp add:zeros_f_def) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
918 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
919 |
show "open (s - zeros_f)" using \<open>finite zeros_f\<close> \<open>open s\<close> finite_imp_closed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
920 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
921 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
922 |
have "((\<lambda>z. 1/z) has_contour_integral 0) (h \<circ> \<gamma>)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
923 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
924 |
have "0 \<notin> path_image (h \<circ> \<gamma>)" using outside_img by (simp add: outside_def) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
925 |
then have "((\<lambda>z. 1/z) has_contour_integral c * winding_number (h \<circ> \<gamma>) 0) (h \<circ> \<gamma>)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
926 |
using has_contour_integral_winding_number[of "h o \<gamma>" 0,simplified] valid_h |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
927 |
unfolding c_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
928 |
moreover have "winding_number (h o \<gamma>) 0 = 0" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
929 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
930 |
have "0 \<in> outside (path_image (h \<circ> \<gamma>))" using outside_img . |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
931 |
moreover have "path (h o \<gamma>)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
932 |
using valid_h by (simp add: valid_path_imp_path) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
933 |
moreover have "pathfinish (h o \<gamma>) = pathstart (h o \<gamma>)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
934 |
by (simp add: loop pathfinish_compose pathstart_compose) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
935 |
ultimately show ?thesis using winding_number_zero_in_outside by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
936 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
937 |
ultimately show ?thesis by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
938 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
939 |
moreover have "vector_derivative (h \<circ> \<gamma>) (at x) = vector_derivative \<gamma> (at x) * deriv h (\<gamma> x)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
940 |
when "x\<in>{0..1} - spikes" for x |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
941 |
proof (rule vector_derivative_chain_at_general) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
942 |
show "\<gamma> differentiable at x" using that \<open>valid_path \<gamma>\<close> spikes by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
943 |
next |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
944 |
define der where "der \<equiv> \<lambda>p. (deriv g p * f p - g p * deriv f p)/(f p * f p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
945 |
define t where "t \<equiv> \<gamma> x" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
946 |
have "f t\<noteq>0" unfolding zeros_f_def t_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
947 |
by (metis DiffD1 image_eqI norm_not_less_zero norm_zero path_defs(4) path_less that) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
948 |
moreover have "t\<in>s" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
949 |
using contra_subsetD path_image_def path_fg t_def that by fastforce |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
950 |
ultimately have "(h has_field_derivative der t) (at t)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
951 |
unfolding h_def der_def using g_holo f_holo \<open>open s\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
952 |
by (auto intro!: holomorphic_derivI derivative_eq_intros) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
953 |
then show "h field_differentiable at (\<gamma> x)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
954 |
unfolding t_def field_differentiable_def by blast |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
955 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
956 |
then have " ((/) 1 has_contour_integral 0) (h \<circ> \<gamma>) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
957 |
= ((\<lambda>x. deriv h x / h x) has_contour_integral 0) \<gamma>" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
958 |
unfolding has_contour_integral |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
959 |
by (force intro!: has_integral_spike_eq[OF negligible_finite, OF \<open>finite spikes\<close>]) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
960 |
ultimately show ?thesis by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
961 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
962 |
then have "contour_integral \<gamma> (\<lambda>x. deriv h x / h x) = 0" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
963 |
using contour_integral_unique by simp |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
964 |
moreover have "contour_integral \<gamma> (\<lambda>x. deriv fg x / fg x) = contour_integral \<gamma> (\<lambda>x. deriv f x / f x) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
965 |
+ contour_integral \<gamma> (\<lambda>p. deriv h p / h p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
966 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
967 |
have "(\<lambda>p. deriv f p / f p) contour_integrable_on \<gamma>" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
968 |
proof (rule contour_integrable_holomorphic_simple[OF _ _ \<open>valid_path \<gamma>\<close> path_f]) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
969 |
show "open (s - zeros_f)" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
970 |
using finite_imp_closed[OF \<open>finite zeros_f\<close>] \<open>open s\<close> by auto |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
971 |
then show "(\<lambda>p. deriv f p / f p) holomorphic_on s - zeros_f" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
972 |
using f_holo |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
973 |
by (auto intro!: holomorphic_intros simp add:zeros_f_def) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
974 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
975 |
moreover have "(\<lambda>p. deriv h p / h p) contour_integrable_on \<gamma>" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
976 |
using h_contour |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
977 |
by (simp add: has_contour_integral_integrable) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
978 |
ultimately have "contour_integral \<gamma> (\<lambda>x. deriv f x / f x + deriv h x / h x) = |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
979 |
contour_integral \<gamma> (\<lambda>p. deriv f p / f p) + contour_integral \<gamma> (\<lambda>p. deriv h p / h p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
980 |
using contour_integral_add[of "(\<lambda>p. deriv f p / f p)" \<gamma> "(\<lambda>p. deriv h p / h p)" ] |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
981 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
982 |
moreover have "deriv fg p / fg p = deriv f p / f p + deriv h p / h p" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
983 |
when "p\<in> path_image \<gamma>" for p |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
984 |
proof - |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
985 |
have "fg p \<noteq> 0" and "f p \<noteq> 0" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
986 |
using path_f path_fg that unfolding zeros_f_def zeros_fg_def by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
987 |
have "h p \<noteq> 0" |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
988 |
proof (rule ccontr) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
989 |
assume "\<not> h p \<noteq> 0" |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
990 |
then have "cmod (g p/f p) = 1" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
991 |
by (simp add: add_eq_0_iff2 h_def) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
992 |
then show False |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
993 |
by (smt (verit) divide_eq_1_iff norm_divide path_less that) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
994 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
995 |
have der_fg:"deriv fg p = deriv f p + deriv g p" unfolding fg_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
996 |
using f_holo g_holo holomorphic_on_imp_differentiable_at[OF _ \<open>open s\<close>] path_img that |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
997 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
998 |
have der_h:"deriv h p = (deriv g p * f p - g p * deriv f p)/(f p * f p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
999 |
proof - |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1000 |
define der where "der \<equiv> \<lambda>p. (deriv g p * f p - g p * deriv f p)/(f p * f p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1001 |
have "p\<in>s" using path_img that by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1002 |
then have "(h has_field_derivative der p) (at p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1003 |
unfolding h_def der_def using g_holo f_holo \<open>open s\<close> \<open>f p\<noteq>0\<close> |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1004 |
by (auto intro!: derivative_eq_intros holomorphic_derivI) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1005 |
then show ?thesis unfolding der_def using DERIV_imp_deriv by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1006 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1007 |
show ?thesis |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1008 |
using \<open>h p\<noteq>0\<close> \<open>f p\<noteq>0\<close> \<open>fg p\<noteq>0\<close> |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1009 |
unfolding der_fg der_h |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1010 |
apply (simp add: divide_simps h_def fg_def) |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1011 |
by (simp add: mult.commute mult.left_commute ring_class.ring_distribs(1)) |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1012 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1013 |
then have "contour_integral \<gamma> (\<lambda>p. deriv fg p / fg p) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1014 |
= contour_integral \<gamma> (\<lambda>p. deriv f p / f p + deriv h p / h p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1015 |
by (elim contour_integral_eq) |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1016 |
ultimately show ?thesis by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1017 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1018 |
moreover have "contour_integral \<gamma> (\<lambda>x. deriv fg x / fg x) = c * (\<Sum>p\<in>zeros_fg. w p * zorder fg p)" |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
1019 |
proof - |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1020 |
have "fg holomorphic_on s" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1021 |
unfolding fg_def using f_holo g_holo holomorphic_on_add by auto |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
1022 |
moreover |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1023 |
have "path_image \<gamma> \<subseteq> s - {p\<in>s. fg p = 0}" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1024 |
using path_fg unfolding zeros_fg_def . |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
1025 |
moreover |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1026 |
have " finite {p\<in>s. fg p = 0}" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1027 |
using \<open>finite zeros_fg\<close> unfolding zeros_fg_def . |
77223
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
1028 |
ultimately show ?thesis |
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
1029 |
unfolding c_def zeros_fg_def w_def |
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
1030 |
using argument_principle[OF \<open>open s\<close> \<open>connected s\<close> _ _ \<open>valid_path \<gamma>\<close> loop _ homo, of _ "{}" "\<lambda>_. 1"] |
607e1e345e8f
Lots of new material chiefly about complex analysis
paulson <lp15@cam.ac.uk>
parents:
73048
diff
changeset
|
1031 |
by simp |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1032 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1033 |
moreover have "contour_integral \<gamma> (\<lambda>x. deriv f x / f x) = c * (\<Sum>p\<in>zeros_f. w p * zorder f p)" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1034 |
unfolding c_def zeros_f_def w_def |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1035 |
proof (rule argument_principle[OF \<open>open s\<close> \<open>connected s\<close> _ _ \<open>valid_path \<gamma>\<close> loop _ homo |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1036 |
, of _ "{}" "\<lambda>_. 1",simplified]) |
78517
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1037 |
show "f holomorphic_on s" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1038 |
using f_holo g_holo holomorphic_on_add by auto |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1039 |
show "path_image \<gamma> \<subseteq> s - {p\<in>s. f p = 0}" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1040 |
using path_f unfolding zeros_f_def . |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1041 |
show " finite {p\<in>s. f p = 0}" |
28c1f4f5335f
Numerous minor tweaks and simplifications
paulson <lp15@cam.ac.uk>
parents:
77322
diff
changeset
|
1042 |
using \<open>finite zeros_f\<close> unfolding zeros_f_def . |
71201
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1043 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1044 |
ultimately have " c* (\<Sum>p\<in>zeros_fg. w p * (zorder fg p)) = c* (\<Sum>p\<in>zeros_f. w p * (zorder f p))" |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1045 |
by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1046 |
then show ?thesis unfolding c_def using w_def by auto |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1047 |
qed |
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1048 |
|
6617fb368a06
Reorganised HOL-Complex_Analysis
Manuel Eberl <eberlm@in.tum.de>
parents:
diff
changeset
|
1049 |
end |