src/HOL/Analysis/Complex_Analysis_Basics.thy
author wenzelm
Mon, 20 Feb 2023 21:40:52 +0100
changeset 77319 87698fe320bb
parent 77226 69956724ad4f
child 78516 56a408fa2440
permissions -rw-r--r--
clarified signature: more robust operations, without assumption about node 0;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
     1
(*  Author: John Harrison, Marco Maggesi, Graziano Gentili, Gianni Ciolli, Valentina Bruno
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
     2
    Ported from "hol_light/Multivariate/canal.ml" by L C Paulson (2014)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
     3
*)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
     4
60420
884f54e01427 isabelle update_cartouches;
wenzelm
parents: 60162
diff changeset
     5
section \<open>Complex Analysis Basics\<close>
71167
b4d409c65a76 Rearrangement of material in Complex_Analysis_Basics, which contained much that had nothing to do with complex analysis.
paulson <lp15@cam.ac.uk>
parents: 71030
diff changeset
     6
text \<open>Definitions of analytic and holomorphic functions, limit theorems, complex differentiation\<close>
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
     7
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
     8
theory Complex_Analysis_Basics
77200
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
     9
  imports Derivative "HOL-Library.Nonpos_Ints" Uncountable_Sets
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
    10
begin
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
    11
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69529
diff changeset
    12
subsection\<^marker>\<open>tag unimportant\<close>\<open>General lemmas\<close>
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
    13
62131
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
    14
lemma nonneg_Reals_cmod_eq_Re: "z \<in> \<real>\<^sub>\<ge>\<^sub>0 \<Longrightarrow> norm z = Re z"
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
    15
  by (simp add: complex_nonneg_Reals_iff cmod_eq_Re)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    16
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
    17
lemma fact_cancel:
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
    18
  fixes c :: "'a::real_field"
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
    19
  shows "of_nat (Suc n) * c / (fact (Suc n)) = c / (fact n)"
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
    20
  using of_nat_neq_0 by force
56889
48a745e1bde7 avoid the Complex constructor, use the more natural Re/Im view; moved csqrt to Complex.
hoelzl
parents: 56479
diff changeset
    21
68721
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    22
lemma vector_derivative_cnj_within:
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    23
  assumes "at x within A \<noteq> bot" and "f differentiable at x within A"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    24
  shows   "vector_derivative (\<lambda>z. cnj (f z)) (at x within A) = 
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    25
             cnj (vector_derivative f (at x within A))" (is "_ = cnj ?D")
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    26
proof -
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    27
  let ?D = "vector_derivative f (at x within A)"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    28
  from assms have "(f has_vector_derivative ?D) (at x within A)"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    29
    by (subst (asm) vector_derivative_works)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    30
  hence "((\<lambda>x. cnj (f x)) has_vector_derivative cnj ?D) (at x within A)"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    31
    by (rule has_vector_derivative_cnj)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    32
  thus ?thesis using assms by (auto dest: vector_derivative_within)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    33
qed
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    34
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    35
lemma vector_derivative_cnj:
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    36
  assumes "f differentiable at x"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    37
  shows   "vector_derivative (\<lambda>z. cnj (f z)) (at x) = cnj (vector_derivative f (at x))"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    38
  using assms by (intro vector_derivative_cnj_within) auto
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
    39
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    40
lemma
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    41
  shows open_halfspace_Re_lt: "open {z. Re(z) < b}"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    42
    and open_halfspace_Re_gt: "open {z. Re(z) > b}"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    43
    and closed_halfspace_Re_ge: "closed {z. Re(z) \<ge> b}"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    44
    and closed_halfspace_Re_le: "closed {z. Re(z) \<le> b}"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    45
    and closed_halfspace_Re_eq: "closed {z. Re(z) = b}"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    46
    and open_halfspace_Im_lt: "open {z. Im(z) < b}"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    47
    and open_halfspace_Im_gt: "open {z. Im(z) > b}"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    48
    and closed_halfspace_Im_ge: "closed {z. Im(z) \<ge> b}"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    49
    and closed_halfspace_Im_le: "closed {z. Im(z) \<le> b}"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    50
    and closed_halfspace_Im_eq: "closed {z. Im(z) = b}"
63332
f164526d8727 move open_Collect_eq/less to HOL
hoelzl
parents: 63092
diff changeset
    51
  by (intro open_Collect_less closed_Collect_le closed_Collect_eq continuous_on_Re
f164526d8727 move open_Collect_eq/less to HOL
hoelzl
parents: 63092
diff changeset
    52
            continuous_on_Im continuous_on_id continuous_on_const)+
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    53
77200
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    54
lemma uncountable_halfspace_Im_gt: "uncountable {z. Im z > c}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    55
proof -
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    56
  obtain r where r: "r > 0" "ball ((c + 1) *\<^sub>R \<i>) r \<subseteq> {z. Im z > c}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    57
    using open_halfspace_Im_gt[of c] unfolding open_contains_ball by force
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    58
  then show ?thesis
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    59
    using countable_subset uncountable_ball by blast
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    60
qed
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    61
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    62
lemma uncountable_halfspace_Im_lt: "uncountable {z. Im z < c}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    63
proof -
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    64
  obtain r where r: "r > 0" "ball ((c - 1) *\<^sub>R \<i>) r \<subseteq> {z. Im z < c}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    65
    using open_halfspace_Im_lt[of c] unfolding open_contains_ball by force
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    66
  then show ?thesis
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    67
    using countable_subset uncountable_ball by blast
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    68
qed
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    69
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    70
lemma uncountable_halfspace_Re_gt: "uncountable {z. Re z > c}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    71
proof -
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    72
  obtain r where r: "r > 0" "ball (of_real(c + 1)) r \<subseteq> {z. Re z > c}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    73
    using open_halfspace_Re_gt[of c] unfolding open_contains_ball by force
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    74
  then show ?thesis
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    75
    using countable_subset uncountable_ball by blast
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    76
qed
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    77
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    78
lemma uncountable_halfspace_Re_lt: "uncountable {z. Re z < c}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    79
proof -
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    80
  obtain r where r: "r > 0" "ball (of_real(c - 1)) r \<subseteq> {z. Re z < c}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    81
    using open_halfspace_Re_lt[of c] unfolding open_contains_ball by force
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    82
  then show ?thesis
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    83
    using countable_subset uncountable_ball by blast
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    84
qed
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    85
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    86
lemma connected_halfspace_Im_gt [intro]: "connected {z. c < Im z}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    87
  by (intro convex_connected convex_halfspace_Im_gt)
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    88
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    89
lemma connected_halfspace_Im_lt [intro]: "connected {z. c > Im z}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    90
  by (intro convex_connected convex_halfspace_Im_lt)
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    91
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    92
lemma connected_halfspace_Re_gt [intro]: "connected {z. c < Re z}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    93
  by (intro convex_connected convex_halfspace_Re_gt)
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    94
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    95
lemma connected_halfspace_Re_lt [intro]: "connected {z. c > Re z}"
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    96
  by (intro convex_connected convex_halfspace_Re_lt)
8f2e6186408f Some more new material and some tidying of existing proofs
paulson <lp15@cam.ac.uk>
parents: 77166
diff changeset
    97
  
61070
b72a990adfe2 prefer symbols;
wenzelm
parents: 60585
diff changeset
    98
lemma closed_complex_Reals: "closed (\<real> :: complex set)"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
    99
proof -
61070
b72a990adfe2 prefer symbols;
wenzelm
parents: 60585
diff changeset
   100
  have "(\<real> :: complex set) = {z. Im z = 0}"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   101
    by (auto simp: complex_is_Real_iff)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   102
  then show ?thesis
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   103
    by (metis closed_halfspace_Im_eq)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   104
qed
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   105
60017
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   106
lemma closed_Real_halfspace_Re_le: "closed (\<real> \<inter> {w. Re w \<le> x})"
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   107
  by (simp add: closed_Int closed_complex_Reals closed_halfspace_Re_le)
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   108
69180
922833cc6839 Tagged some theories in HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 69064
diff changeset
   109
lemma closed_nonpos_Reals_complex [simp]: "closed (\<real>\<^sub>\<le>\<^sub>0 :: complex set)"
62131
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   110
proof -
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   111
  have "\<real>\<^sub>\<le>\<^sub>0 = \<real> \<inter> {z. Re(z) \<le> 0}"
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   112
    using complex_nonpos_Reals_iff complex_is_Real_iff by auto
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   113
  then show ?thesis
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   114
    by (metis closed_Real_halfspace_Re_le)
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   115
qed
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   116
60017
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   117
lemma closed_Real_halfspace_Re_ge: "closed (\<real> \<inter> {w. x \<le> Re(w)})"
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   118
  using closed_halfspace_Re_ge
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   119
  by (simp add: closed_Int closed_complex_Reals)
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   120
69180
922833cc6839 Tagged some theories in HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 69064
diff changeset
   121
lemma closed_nonneg_Reals_complex [simp]: "closed (\<real>\<^sub>\<ge>\<^sub>0 :: complex set)"
62131
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   122
proof -
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   123
  have "\<real>\<^sub>\<ge>\<^sub>0 = \<real> \<inter> {z. Re(z) \<ge> 0}"
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   124
    using complex_nonneg_Reals_iff complex_is_Real_iff by auto
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   125
  then show ?thesis
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   126
    by (metis closed_Real_halfspace_Re_ge)
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   127
qed
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   128
60017
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   129
lemma closed_real_abs_le: "closed {w \<in> \<real>. \<bar>Re w\<bar> \<le> r}"
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   130
proof -
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   131
  have "{w \<in> \<real>. \<bar>Re w\<bar> \<le> r} = (\<real> \<inter> {w. Re w \<le> r}) \<inter> (\<real> \<inter> {w. Re w \<ge> -r})"
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   132
    by auto
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   133
  then show "closed {w \<in> \<real>. \<bar>Re w\<bar> \<le> r}"
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   134
    by (simp add: closed_Int closed_Real_halfspace_Re_ge closed_Real_halfspace_Re_le)
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   135
qed
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
   136
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   137
lemma real_lim:
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   138
  fixes l::complex
69508
2a4c8a2a3f8e tuned headers; ~ -> \<not>
nipkow
parents: 69286
diff changeset
   139
  assumes "(f \<longlongrightarrow> l) F" and "\<not> trivial_limit F" and "eventually P F" and "\<And>a. P a \<Longrightarrow> f a \<in> \<real>"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   140
  shows  "l \<in> \<real>"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   141
proof (rule Lim_in_closed_set[OF closed_complex_Reals _ assms(2,1)])
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   142
  show "eventually (\<lambda>x. f x \<in> \<real>) F"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   143
    using assms(3, 4) by (auto intro: eventually_mono)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   144
qed
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   145
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   146
lemma real_lim_sequentially:
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   147
  fixes l::complex
61973
0c7e865fa7cb more symbols;
wenzelm
parents: 61969
diff changeset
   148
  shows "(f \<longlongrightarrow> l) sequentially \<Longrightarrow> (\<exists>N. \<forall>n\<ge>N. f n \<in> \<real>) \<Longrightarrow> l \<in> \<real>"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   149
by (rule real_lim [where F=sequentially]) (auto simp: eventually_sequentially)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   150
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   151
lemma real_series:
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   152
  fixes l::complex
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   153
  shows "f sums l \<Longrightarrow> (\<And>n. f n \<in> \<real>) \<Longrightarrow> l \<in> \<real>"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   154
unfolding sums_def
64267
b9a1486e79be setsum -> sum
nipkow
parents: 63941
diff changeset
   155
by (metis real_lim_sequentially sum_in_Reals)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   156
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   157
lemma Lim_null_comparison_Re:
61973
0c7e865fa7cb more symbols;
wenzelm
parents: 61969
diff changeset
   158
  assumes "eventually (\<lambda>x. norm(f x) \<le> Re(g x)) F" "(g \<longlongrightarrow> 0) F" shows "(f \<longlongrightarrow> 0) F"
56889
48a745e1bde7 avoid the Complex constructor, use the more natural Re/Im view; moved csqrt to Complex.
hoelzl
parents: 56479
diff changeset
   159
  by (rule Lim_null_comparison[OF assms(1)] tendsto_eq_intros assms(2))+ simp
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   160
60420
884f54e01427 isabelle update_cartouches;
wenzelm
parents: 60162
diff changeset
   161
subsection\<open>Holomorphic functions\<close>
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   162
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69529
diff changeset
   163
definition\<^marker>\<open>tag important\<close> holomorphic_on :: "[complex \<Rightarrow> complex, complex set] \<Rightarrow> bool"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   164
           (infixl "(holomorphic'_on)" 50)
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   165
  where "f holomorphic_on s \<equiv> \<forall>x\<in>s. f field_differentiable (at x within s)"
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   166
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69529
diff changeset
   167
named_theorems\<^marker>\<open>tag important\<close> holomorphic_intros "structural introduction rules for holomorphic_on"
61520
8f85bb443d33 Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents: 61518
diff changeset
   168
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   169
lemma holomorphic_onI [intro?]: "(\<And>x. x \<in> s \<Longrightarrow> f field_differentiable (at x within s)) \<Longrightarrow> f holomorphic_on s"
62131
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   170
  by (simp add: holomorphic_on_def)
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   171
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   172
lemma holomorphic_onD [dest?]: "\<lbrakk>f holomorphic_on s; x \<in> s\<rbrakk> \<Longrightarrow> f field_differentiable (at x within s)"
62131
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   173
  by (simp add: holomorphic_on_def)
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   174
64394
141e1ed8d5a0 more new material
paulson <lp15@cam.ac.uk>
parents: 64267
diff changeset
   175
lemma holomorphic_on_imp_differentiable_on:
141e1ed8d5a0 more new material
paulson <lp15@cam.ac.uk>
parents: 64267
diff changeset
   176
    "f holomorphic_on s \<Longrightarrow> f differentiable_on s"
141e1ed8d5a0 more new material
paulson <lp15@cam.ac.uk>
parents: 64267
diff changeset
   177
  unfolding holomorphic_on_def differentiable_on_def
141e1ed8d5a0 more new material
paulson <lp15@cam.ac.uk>
parents: 64267
diff changeset
   178
  by (simp add: field_differentiable_imp_differentiable)
141e1ed8d5a0 more new material
paulson <lp15@cam.ac.uk>
parents: 64267
diff changeset
   179
62131
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   180
lemma holomorphic_on_imp_differentiable_at:
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   181
   "\<lbrakk>f holomorphic_on s; open s; x \<in> s\<rbrakk> \<Longrightarrow> f field_differentiable (at x)"
62131
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   182
using at_within_open holomorphic_on_def by fastforce
1baed43f453e nonneg_Reals, nonpos_Reals, Cauchy integral formula, etc.
paulson
parents: 62087
diff changeset
   183
61520
8f85bb443d33 Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents: 61518
diff changeset
   184
lemma holomorphic_on_empty [holomorphic_intros]: "f holomorphic_on {}"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   185
  by (simp add: holomorphic_on_def)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   186
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   187
lemma holomorphic_on_open:
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   188
    "open s \<Longrightarrow> f holomorphic_on s \<longleftrightarrow> (\<forall>x \<in> s. \<exists>f'. DERIV f x :> f')"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   189
  by (auto simp: holomorphic_on_def field_differentiable_def has_field_derivative_def at_within_open [of _ s])
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   190
74513
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   191
lemma holomorphic_on_UN_open:
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   192
  assumes "\<And>n. n \<in> I \<Longrightarrow> f holomorphic_on A n" "\<And>n. n \<in> I \<Longrightarrow> open (A n)"
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   193
  shows   "f holomorphic_on (\<Union>n\<in>I. A n)"
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   194
proof -
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   195
  have "f field_differentiable at z within (\<Union>n\<in>I. A n)" if "z \<in> (\<Union>n\<in>I. A n)" for z
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   196
  proof -
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   197
    from that obtain n where "n \<in> I" "z \<in> A n"
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   198
      by blast
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   199
    hence "f holomorphic_on A n" "open (A n)"
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   200
      by (simp add: assms)+
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   201
    with \<open>z \<in> A n\<close> have "f field_differentiable at z"
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   202
      by (auto simp: holomorphic_on_open field_differentiable_def)
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   203
    thus ?thesis
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   204
      by (meson field_differentiable_at_within)
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   205
  qed
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   206
  thus ?thesis
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   207
    by (auto simp: holomorphic_on_def)
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   208
qed
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   209
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   210
lemma holomorphic_on_imp_continuous_on:
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   211
    "f holomorphic_on s \<Longrightarrow> continuous_on s f"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   212
  by (metis field_differentiable_imp_continuous_at continuous_on_eq_continuous_within holomorphic_on_def)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   213
73885
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   214
lemma holomorphic_closedin_preimage_constant:
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   215
  assumes "f holomorphic_on D" 
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   216
  shows "closedin (top_of_set D) {z\<in>D. f z = a}"
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   217
  by (simp add: assms continuous_closedin_preimage_constant holomorphic_on_imp_continuous_on)
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   218
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   219
lemma holomorphic_closed_preimage_constant:
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   220
  assumes "f holomorphic_on UNIV" 
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   221
  shows "closed {z. f z = a}"
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   222
  using holomorphic_closedin_preimage_constant [OF assms] by simp
26171a89466a A few useful lemmas about derivatives, colinearity and other topics
paulson <lp15@cam.ac.uk>
parents: 71633
diff changeset
   223
62540
f2fc5485e3b0 Wenda Li's new material: residue theorem, argument_principle, Rouche_theorem
paulson <lp15@cam.ac.uk>
parents: 62534
diff changeset
   224
lemma holomorphic_on_subset [elim]:
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   225
    "f holomorphic_on s \<Longrightarrow> t \<subseteq> s \<Longrightarrow> f holomorphic_on t"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   226
  unfolding holomorphic_on_def
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   227
  by (metis field_differentiable_within_subset subsetD)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   228
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   229
lemma holomorphic_transform: "\<lbrakk>f holomorphic_on s; \<And>x. x \<in> s \<Longrightarrow> f x = g x\<rbrakk> \<Longrightarrow> g holomorphic_on s"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   230
  by (metis field_differentiable_transform_within linordered_field_no_ub holomorphic_on_def)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   231
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   232
lemma holomorphic_cong: "s = t ==> (\<And>x. x \<in> s \<Longrightarrow> f x = g x) \<Longrightarrow> f holomorphic_on s \<longleftrightarrow> g holomorphic_on t"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   233
  by (metis holomorphic_transform)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   234
69064
5840724b1d71 Prefix form of infix with * on either side no longer needs special treatment
nipkow
parents: 68721
diff changeset
   235
lemma holomorphic_on_linear [simp, holomorphic_intros]: "((*) c) holomorphic_on s"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   236
  unfolding holomorphic_on_def by (metis field_differentiable_linear)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   237
62217
527488dc8b90 Reorganised a huge proof
paulson <lp15@cam.ac.uk>
parents: 62131
diff changeset
   238
lemma holomorphic_on_const [simp, holomorphic_intros]: "(\<lambda>z. c) holomorphic_on s"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   239
  unfolding holomorphic_on_def by (metis field_differentiable_const)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   240
62217
527488dc8b90 Reorganised a huge proof
paulson <lp15@cam.ac.uk>
parents: 62131
diff changeset
   241
lemma holomorphic_on_ident [simp, holomorphic_intros]: "(\<lambda>x. x) holomorphic_on s"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   242
  unfolding holomorphic_on_def by (metis field_differentiable_ident)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   243
62217
527488dc8b90 Reorganised a huge proof
paulson <lp15@cam.ac.uk>
parents: 62131
diff changeset
   244
lemma holomorphic_on_id [simp, holomorphic_intros]: "id holomorphic_on s"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   245
  unfolding id_def by (rule holomorphic_on_ident)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   246
74513
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   247
lemma constant_on_imp_holomorphic_on:
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   248
  assumes "f constant_on A"
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   249
  shows   "f holomorphic_on A"
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   250
proof -
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   251
  from assms obtain c where c: "\<forall>x\<in>A. f x = c"
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   252
    unfolding constant_on_def by blast
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   253
  have "f holomorphic_on A \<longleftrightarrow> (\<lambda>_. c) holomorphic_on A"
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   254
    by (intro holomorphic_cong) (use c in auto)
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   255
  thus ?thesis
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   256
    by simp
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   257
qed
67d87d224e00 A few new lemmas plus some refinements
paulson <lp15@cam.ac.uk>
parents: 73885
diff changeset
   258
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   259
lemma holomorphic_on_compose:
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   260
  "f holomorphic_on s \<Longrightarrow> g holomorphic_on (f ` s) \<Longrightarrow> (g o f) holomorphic_on s"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   261
  using field_differentiable_compose_within[of f _ s g]
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   262
  by (auto simp: holomorphic_on_def)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   263
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   264
lemma holomorphic_on_compose_gen:
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   265
  "f holomorphic_on s \<Longrightarrow> g holomorphic_on t \<Longrightarrow> f ` s \<subseteq> t \<Longrightarrow> (g o f) holomorphic_on s"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   266
  by (metis holomorphic_on_compose holomorphic_on_subset)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   267
68721
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   268
lemma holomorphic_on_balls_imp_entire:
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   269
  assumes "\<not>bdd_above A" "\<And>r. r \<in> A \<Longrightarrow> f holomorphic_on ball c r"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   270
  shows   "f holomorphic_on B"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   271
proof (rule holomorphic_on_subset)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   272
  show "f holomorphic_on UNIV" unfolding holomorphic_on_def
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   273
  proof
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   274
    fix z :: complex
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   275
    from \<open>\<not>bdd_above A\<close> obtain r where r: "r \<in> A" "r > norm (z - c)"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   276
      by (meson bdd_aboveI not_le)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   277
    with assms(2) have "f holomorphic_on ball c r" by blast
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   278
    moreover from r have "z \<in> ball c r" by (auto simp: dist_norm norm_minus_commute)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   279
    ultimately show "f field_differentiable at z"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   280
      by (auto simp: holomorphic_on_def at_within_open[of _ "ball c r"])
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   281
  qed
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   282
qed auto
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   283
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   284
lemma holomorphic_on_balls_imp_entire':
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   285
  assumes "\<And>r. r > 0 \<Longrightarrow> f holomorphic_on ball c r"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   286
  shows   "f holomorphic_on B"
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   287
proof (rule holomorphic_on_balls_imp_entire)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   288
  {
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   289
    fix M :: real
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   290
    have "\<exists>x. x > max M 0" by (intro gt_ex)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   291
    hence "\<exists>x>0. x > M" by auto
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   292
  }
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   293
  thus "\<not>bdd_above {(0::real)<..}" unfolding bdd_above_def
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   294
    by (auto simp: not_le)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   295
qed (insert assms, auto)
53ad5c01be3f Small lemmas about analysis
eberlm <eberlm@in.tum.de>
parents: 68296
diff changeset
   296
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   297
lemma holomorphic_on_minus [holomorphic_intros]: "f holomorphic_on A \<Longrightarrow> (\<lambda>z. -(f z)) holomorphic_on A"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   298
  by (metis field_differentiable_minus holomorphic_on_def)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   299
61520
8f85bb443d33 Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents: 61518
diff changeset
   300
lemma holomorphic_on_add [holomorphic_intros]:
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   301
  "\<lbrakk>f holomorphic_on A; g holomorphic_on A\<rbrakk> \<Longrightarrow> (\<lambda>z. f z + g z) holomorphic_on A"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   302
  unfolding holomorphic_on_def by (metis field_differentiable_add)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   303
61520
8f85bb443d33 Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents: 61518
diff changeset
   304
lemma holomorphic_on_diff [holomorphic_intros]:
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   305
  "\<lbrakk>f holomorphic_on A; g holomorphic_on A\<rbrakk> \<Longrightarrow> (\<lambda>z. f z - g z) holomorphic_on A"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   306
  unfolding holomorphic_on_def by (metis field_differentiable_diff)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   307
61520
8f85bb443d33 Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents: 61518
diff changeset
   308
lemma holomorphic_on_mult [holomorphic_intros]:
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   309
  "\<lbrakk>f holomorphic_on A; g holomorphic_on A\<rbrakk> \<Longrightarrow> (\<lambda>z. f z * g z) holomorphic_on A"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   310
  unfolding holomorphic_on_def by (metis field_differentiable_mult)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   311
61520
8f85bb443d33 Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents: 61518
diff changeset
   312
lemma holomorphic_on_inverse [holomorphic_intros]:
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   313
  "\<lbrakk>f holomorphic_on A; \<And>z. z \<in> A \<Longrightarrow> f z \<noteq> 0\<rbrakk> \<Longrightarrow> (\<lambda>z. inverse (f z)) holomorphic_on A"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   314
  unfolding holomorphic_on_def by (metis field_differentiable_inverse)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   315
61520
8f85bb443d33 Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents: 61518
diff changeset
   316
lemma holomorphic_on_divide [holomorphic_intros]:
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   317
  "\<lbrakk>f holomorphic_on A; g holomorphic_on A; \<And>z. z \<in> A \<Longrightarrow> g z \<noteq> 0\<rbrakk> \<Longrightarrow> (\<lambda>z. f z / g z) holomorphic_on A"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   318
  unfolding holomorphic_on_def by (metis field_differentiable_divide)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   319
61520
8f85bb443d33 Cauchy's integral formula, required lemmas, and a bit of reorganisation
paulson <lp15@cam.ac.uk>
parents: 61518
diff changeset
   320
lemma holomorphic_on_power [holomorphic_intros]:
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   321
  "f holomorphic_on A \<Longrightarrow> (\<lambda>z. (f z)^n) holomorphic_on A"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   322
  unfolding holomorphic_on_def by (metis field_differentiable_power)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   323
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   324
lemma holomorphic_on_power_int [holomorphic_intros]:
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   325
  assumes nz: "n \<ge> 0 \<or> (\<forall>x\<in>A. f x \<noteq> 0)" and f: "f holomorphic_on A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   326
  shows   "(\<lambda>x. f x powi n) holomorphic_on A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   327
proof (cases "n \<ge> 0")
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   328
  case True
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   329
  have "(\<lambda>x. f x ^ nat n) holomorphic_on A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   330
    by (simp add: f holomorphic_on_power)
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   331
  with True show ?thesis
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   332
    by (simp add: power_int_def)
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   333
next
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   334
  case False
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   335
  hence "(\<lambda>x. inverse (f x ^ nat (-n))) holomorphic_on A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   336
    using nz by (auto intro!: holomorphic_intros f)
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   337
  with False show ?thesis
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   338
    by (simp add: power_int_def power_inverse)
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   339
qed
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   340
64267
b9a1486e79be setsum -> sum
nipkow
parents: 63941
diff changeset
   341
lemma holomorphic_on_sum [holomorphic_intros]:
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   342
  "(\<And>i. i \<in> I \<Longrightarrow> (f i) holomorphic_on A) \<Longrightarrow> (\<lambda>x. sum (\<lambda>i. f i x) I) holomorphic_on A"
64267
b9a1486e79be setsum -> sum
nipkow
parents: 63941
diff changeset
   343
  unfolding holomorphic_on_def by (metis field_differentiable_sum)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   344
67135
1a94352812f4 Moved material from AFP to Analysis/Number_Theory
Manuel Eberl <eberlm@in.tum.de>
parents: 66827
diff changeset
   345
lemma holomorphic_on_prod [holomorphic_intros]:
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   346
  "(\<And>i. i \<in> I \<Longrightarrow> (f i) holomorphic_on A) \<Longrightarrow> (\<lambda>x. prod (\<lambda>i. f i x) I) holomorphic_on A"
67135
1a94352812f4 Moved material from AFP to Analysis/Number_Theory
Manuel Eberl <eberlm@in.tum.de>
parents: 66827
diff changeset
   347
  by (induction I rule: infinite_finite_induct) (auto intro: holomorphic_intros)
1a94352812f4 Moved material from AFP to Analysis/Number_Theory
Manuel Eberl <eberlm@in.tum.de>
parents: 66827
diff changeset
   348
66486
ffaaa83543b2 Lemmas about analysis and permutations
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   349
lemma holomorphic_pochhammer [holomorphic_intros]:
ffaaa83543b2 Lemmas about analysis and permutations
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   350
  "f holomorphic_on A \<Longrightarrow> (\<lambda>s. pochhammer (f s) n) holomorphic_on A"
ffaaa83543b2 Lemmas about analysis and permutations
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   351
  by (induction n) (auto intro!: holomorphic_intros simp: pochhammer_Suc)
ffaaa83543b2 Lemmas about analysis and permutations
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   352
ffaaa83543b2 Lemmas about analysis and permutations
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   353
lemma holomorphic_on_scaleR [holomorphic_intros]:
ffaaa83543b2 Lemmas about analysis and permutations
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   354
  "f holomorphic_on A \<Longrightarrow> (\<lambda>x. c *\<^sub>R f x) holomorphic_on A"
ffaaa83543b2 Lemmas about analysis and permutations
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   355
  by (auto simp: scaleR_conv_of_real intro!: holomorphic_intros)
ffaaa83543b2 Lemmas about analysis and permutations
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   356
67167
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   357
lemma holomorphic_on_Un [holomorphic_intros]:
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   358
  assumes "f holomorphic_on A" "f holomorphic_on B" "open A" "open B"
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   359
  shows   "f holomorphic_on (A \<union> B)"
68239
0764ee22a4d1 tidy up of Derivative
paulson <lp15@cam.ac.uk>
parents: 68055
diff changeset
   360
  using assms by (auto simp: holomorphic_on_def  at_within_open[of _ A]
67167
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   361
                             at_within_open[of _ B]  at_within_open[of _ "A \<union> B"] open_Un)
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   362
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   363
lemma holomorphic_on_If_Un [holomorphic_intros]:
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   364
  assumes "f holomorphic_on A" "g holomorphic_on B" "open A" "open B"
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   365
  assumes "\<And>z. z \<in> A \<Longrightarrow> z \<in> B \<Longrightarrow> f z = g z"
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   366
  shows   "(\<lambda>z. if z \<in> A then f z else g z) holomorphic_on (A \<union> B)" (is "?h holomorphic_on _")
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   367
proof (intro holomorphic_on_Un)
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   368
  note \<open>f holomorphic_on A\<close>
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   369
  also have "f holomorphic_on A \<longleftrightarrow> ?h holomorphic_on A"
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   370
    by (intro holomorphic_cong) auto
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   371
  finally show \<dots> .
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   372
next
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   373
  note \<open>g holomorphic_on B\<close>
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   374
  also have "g holomorphic_on B \<longleftrightarrow> ?h holomorphic_on B"
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   375
    using assms by (intro holomorphic_cong) auto
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   376
  finally show \<dots> .
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   377
qed (insert assms, auto)
88d1c9d86f48 Moved analysis material from AFP
Manuel Eberl <eberlm@in.tum.de>
parents: 67135
diff changeset
   378
62533
bc25f3916a99 new material to Blochj's theorem, as well as supporting lemmas
paulson <lp15@cam.ac.uk>
parents: 62408
diff changeset
   379
lemma holomorphic_derivI:
bc25f3916a99 new material to Blochj's theorem, as well as supporting lemmas
paulson <lp15@cam.ac.uk>
parents: 62408
diff changeset
   380
     "\<lbrakk>f holomorphic_on S; open S; x \<in> S\<rbrakk>
bc25f3916a99 new material to Blochj's theorem, as well as supporting lemmas
paulson <lp15@cam.ac.uk>
parents: 62408
diff changeset
   381
      \<Longrightarrow> (f has_field_derivative deriv f x) (at x within T)"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   382
by (metis DERIV_deriv_iff_field_differentiable at_within_open  holomorphic_on_def has_field_derivative_at_within)
62533
bc25f3916a99 new material to Blochj's theorem, as well as supporting lemmas
paulson <lp15@cam.ac.uk>
parents: 62408
diff changeset
   383
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   384
lemma complex_derivative_transform_within_open:
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   385
  "\<lbrakk>f holomorphic_on s; g holomorphic_on s; open s; z \<in> s; \<And>w. w \<in> s \<Longrightarrow> f w = g w\<rbrakk>
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   386
   \<Longrightarrow> deriv f z = deriv g z"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   387
  unfolding holomorphic_on_def
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   388
  by (rule DERIV_imp_deriv)
71029
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 71001
diff changeset
   389
     (metis DERIV_deriv_iff_field_differentiable has_field_derivative_transform_within_open at_within_open)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   390
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   391
lemma holomorphic_on_compose_cnj_cnj:
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   392
  assumes "f holomorphic_on cnj ` A" "open A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   393
  shows   "cnj \<circ> f \<circ> cnj holomorphic_on A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   394
proof -
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   395
  have [simp]: "open (cnj ` A)"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   396
    unfolding image_cnj_conv_vimage_cnj using assms by (intro open_vimage) auto
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   397
  show ?thesis
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   398
    using assms unfolding holomorphic_on_def
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   399
    by (auto intro!: field_differentiable_cnj_cnj simp: at_within_open_NO_MATCH)
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   400
qed
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   401
  
62533
bc25f3916a99 new material to Blochj's theorem, as well as supporting lemmas
paulson <lp15@cam.ac.uk>
parents: 62408
diff changeset
   402
lemma holomorphic_nonconstant:
bc25f3916a99 new material to Blochj's theorem, as well as supporting lemmas
paulson <lp15@cam.ac.uk>
parents: 62408
diff changeset
   403
  assumes holf: "f holomorphic_on S" and "open S" "\<xi> \<in> S" "deriv f \<xi> \<noteq> 0"
bc25f3916a99 new material to Blochj's theorem, as well as supporting lemmas
paulson <lp15@cam.ac.uk>
parents: 62408
diff changeset
   404
    shows "\<not> f constant_on S"
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   405
  by (rule nonzero_deriv_nonconstant [of f "deriv f \<xi>" \<xi> S])
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   406
    (use assms in \<open>auto simp: holomorphic_derivI\<close>)
62533
bc25f3916a99 new material to Blochj's theorem, as well as supporting lemmas
paulson <lp15@cam.ac.uk>
parents: 62408
diff changeset
   407
60420
884f54e01427 isabelle update_cartouches;
wenzelm
parents: 60162
diff changeset
   408
subsection\<open>Analyticity on a set\<close>
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   409
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69529
diff changeset
   410
definition\<^marker>\<open>tag important\<close> analytic_on (infixl "(analytic'_on)" 50)
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   411
  where "f analytic_on S \<equiv> \<forall>x \<in> S. \<exists>e. 0 < e \<and> f holomorphic_on (ball x e)"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   412
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69529
diff changeset
   413
named_theorems\<^marker>\<open>tag important\<close> analytic_intros "introduction rules for proving analyticity"
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   414
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   415
lemma analytic_imp_holomorphic: "f analytic_on S \<Longrightarrow> f holomorphic_on S"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   416
  by (simp add: at_within_open [OF _ open_ball] analytic_on_def holomorphic_on_def)
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   417
     (metis centre_in_ball field_differentiable_at_within)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   418
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   419
lemma analytic_on_open: "open S \<Longrightarrow> f analytic_on S \<longleftrightarrow> f holomorphic_on S"
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   420
  by (meson analytic_imp_holomorphic analytic_on_def holomorphic_on_subset openE)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   421
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   422
lemma analytic_on_imp_differentiable_at:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   423
  "f analytic_on S \<Longrightarrow> x \<in> S \<Longrightarrow> f field_differentiable (at x)"
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   424
  using analytic_on_def holomorphic_on_imp_differentiable_at by auto
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   425
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   426
lemma analytic_at_imp_isCont:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   427
  assumes "f analytic_on {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   428
  shows   "isCont f z"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   429
  using assms by (meson analytic_on_imp_differentiable_at field_differentiable_imp_continuous_at insertI1)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   430
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   431
lemma analytic_at_neq_imp_eventually_neq:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   432
  assumes "f analytic_on {x}" "f x \<noteq> c"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   433
  shows   "eventually (\<lambda>y. f y \<noteq> c) (at x)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   434
proof (intro tendsto_imp_eventually_ne)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   435
  show "f \<midarrow>x\<rightarrow> f x"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   436
    using assms by (simp add: analytic_at_imp_isCont isContD)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   437
qed (use assms in auto)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   438
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   439
lemma analytic_on_subset: "f analytic_on S \<Longrightarrow> T \<subseteq> S \<Longrightarrow> f analytic_on T"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   440
  by (auto simp: analytic_on_def)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   441
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   442
lemma analytic_on_Un: "f analytic_on (S \<union> T) \<longleftrightarrow> f analytic_on S \<and> f analytic_on T"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   443
  by (auto simp: analytic_on_def)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   444
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   445
lemma analytic_on_Union: "f analytic_on (\<Union>\<T>) \<longleftrightarrow> (\<forall>T \<in> \<T>. f analytic_on T)"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   446
  by (auto simp: analytic_on_def)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   447
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   448
lemma analytic_on_UN: "f analytic_on (\<Union>i\<in>I. S i) \<longleftrightarrow> (\<forall>i\<in>I. f analytic_on (S i))"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   449
  by (auto simp: analytic_on_def)
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   450
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   451
lemma analytic_on_holomorphic:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   452
  "f analytic_on S \<longleftrightarrow> (\<exists>T. open T \<and> S \<subseteq> T \<and> f holomorphic_on T)"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   453
  (is "?lhs = ?rhs")
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   454
proof -
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   455
  have "?lhs \<longleftrightarrow> (\<exists>T. open T \<and> S \<subseteq> T \<and> f analytic_on T)"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   456
  proof safe
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   457
    assume "f analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   458
    then show "\<exists>T. open T \<and> S \<subseteq> T \<and> f analytic_on T"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   459
      apply (simp add: analytic_on_def)
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   460
      apply (rule exI [where x="\<Union>{U. open U \<and> f analytic_on U}"], auto)
66827
c94531b5007d Divided Topology_Euclidean_Space in two, creating new theory Connected. Also deleted some duplicate / variant theorems
paulson <lp15@cam.ac.uk>
parents: 66486
diff changeset
   461
      apply (metis open_ball analytic_on_open centre_in_ball)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   462
      by (metis analytic_on_def)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   463
  next
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   464
    fix T
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   465
    assume "open T" "S \<subseteq> T" "f analytic_on T"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   466
    then show "f analytic_on S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   467
        by (metis analytic_on_subset)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   468
  qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   469
  also have "... \<longleftrightarrow> ?rhs"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   470
    by (auto simp: analytic_on_open)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   471
  finally show ?thesis .
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   472
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   473
69064
5840724b1d71 Prefix form of infix with * on either side no longer needs special treatment
nipkow
parents: 68721
diff changeset
   474
lemma analytic_on_linear [analytic_intros,simp]: "((*) c) analytic_on S"
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   475
  by (auto simp add: analytic_on_holomorphic)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   476
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   477
lemma analytic_on_const [analytic_intros,simp]: "(\<lambda>z. c) analytic_on S"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   478
  by (metis analytic_on_def holomorphic_on_const zero_less_one)
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   479
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   480
lemma analytic_on_ident [analytic_intros,simp]: "(\<lambda>x. x) analytic_on S"
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   481
  by (simp add: analytic_on_def gt_ex)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   482
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   483
lemma analytic_on_id [analytic_intros]: "id analytic_on S"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   484
  unfolding id_def by (rule analytic_on_ident)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   485
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   486
lemma analytic_on_compose:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   487
  assumes f: "f analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   488
      and g: "g analytic_on (f ` S)"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   489
    shows "(g o f) analytic_on S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   490
unfolding analytic_on_def
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   491
proof (intro ballI)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   492
  fix x
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   493
  assume x: "x \<in> S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   494
  then obtain e where e: "0 < e" and fh: "f holomorphic_on ball x e" using f
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   495
    by (metis analytic_on_def)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   496
  obtain e' where e': "0 < e'" and gh: "g holomorphic_on ball (f x) e'" using g
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   497
    by (metis analytic_on_def g image_eqI x)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   498
  have "isCont f x"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   499
    by (metis analytic_on_imp_differentiable_at field_differentiable_imp_continuous_at f x)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   500
  with e' obtain d where d: "0 < d" and fd: "f ` ball x d \<subseteq> ball (f x) e'"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   501
     by (auto simp: continuous_at_ball)
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   502
  have "g \<circ> f holomorphic_on ball x (min d e)"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   503
    apply (rule holomorphic_on_compose)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   504
    apply (metis fh holomorphic_on_subset min.bounded_iff order_refl subset_ball)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   505
    by (metis fd gh holomorphic_on_subset image_mono min.cobounded1 subset_ball)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   506
  then show "\<exists>e>0. g \<circ> f holomorphic_on ball x e"
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   507
    by (metis d e min_less_iff_conj)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   508
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   509
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   510
lemma analytic_on_compose_gen:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   511
  "f analytic_on S \<Longrightarrow> g analytic_on T \<Longrightarrow> (\<And>z. z \<in> S \<Longrightarrow> f z \<in> T)
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   512
             \<Longrightarrow> g o f analytic_on S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   513
by (metis analytic_on_compose analytic_on_subset image_subset_iff)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   514
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   515
lemma analytic_on_neg [analytic_intros]:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   516
  "f analytic_on S \<Longrightarrow> (\<lambda>z. -(f z)) analytic_on S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   517
by (metis analytic_on_holomorphic holomorphic_on_minus)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   518
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   519
lemma analytic_on_add [analytic_intros]:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   520
  assumes f: "f analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   521
      and g: "g analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   522
    shows "(\<lambda>z. f z + g z) analytic_on S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   523
unfolding analytic_on_def
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   524
proof (intro ballI)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   525
  fix z
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   526
  assume z: "z \<in> S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   527
  then obtain e where e: "0 < e" and fh: "f holomorphic_on ball z e" using f
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   528
    by (metis analytic_on_def)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   529
  obtain e' where e': "0 < e'" and gh: "g holomorphic_on ball z e'" using g
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   530
    by (metis analytic_on_def g z)
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   531
  have "(\<lambda>z. f z + g z) holomorphic_on ball z (min e e')"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   532
    apply (rule holomorphic_on_add)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   533
    apply (metis fh holomorphic_on_subset min.bounded_iff order_refl subset_ball)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   534
    by (metis gh holomorphic_on_subset min.bounded_iff order_refl subset_ball)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   535
  then show "\<exists>e>0. (\<lambda>z. f z + g z) holomorphic_on ball z e"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   536
    by (metis e e' min_less_iff_conj)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   537
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   538
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   539
lemma analytic_on_diff [analytic_intros]:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   540
  assumes f: "f analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   541
      and g: "g analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   542
    shows "(\<lambda>z. f z - g z) analytic_on S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   543
unfolding analytic_on_def
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   544
proof (intro ballI)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   545
  fix z
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   546
  assume z: "z \<in> S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   547
  then obtain e where e: "0 < e" and fh: "f holomorphic_on ball z e" using f
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   548
    by (metis analytic_on_def)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   549
  obtain e' where e': "0 < e'" and gh: "g holomorphic_on ball z e'" using g
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   550
    by (metis analytic_on_def g z)
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   551
  have "(\<lambda>z. f z - g z) holomorphic_on ball z (min e e')"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   552
    apply (rule holomorphic_on_diff)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   553
    apply (metis fh holomorphic_on_subset min.bounded_iff order_refl subset_ball)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   554
    by (metis gh holomorphic_on_subset min.bounded_iff order_refl subset_ball)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   555
  then show "\<exists>e>0. (\<lambda>z. f z - g z) holomorphic_on ball z e"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   556
    by (metis e e' min_less_iff_conj)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   557
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   558
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   559
lemma analytic_on_mult [analytic_intros]:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   560
  assumes f: "f analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   561
      and g: "g analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   562
    shows "(\<lambda>z. f z * g z) analytic_on S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   563
unfolding analytic_on_def
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   564
proof (intro ballI)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   565
  fix z
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   566
  assume z: "z \<in> S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   567
  then obtain e where e: "0 < e" and fh: "f holomorphic_on ball z e" using f
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   568
    by (metis analytic_on_def)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   569
  obtain e' where e': "0 < e'" and gh: "g holomorphic_on ball z e'" using g
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   570
    by (metis analytic_on_def g z)
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   571
  have "(\<lambda>z. f z * g z) holomorphic_on ball z (min e e')"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   572
    apply (rule holomorphic_on_mult)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   573
    apply (metis fh holomorphic_on_subset min.bounded_iff order_refl subset_ball)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   574
    by (metis gh holomorphic_on_subset min.bounded_iff order_refl subset_ball)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   575
  then show "\<exists>e>0. (\<lambda>z. f z * g z) holomorphic_on ball z e"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   576
    by (metis e e' min_less_iff_conj)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   577
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   578
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   579
lemma analytic_on_inverse [analytic_intros]:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   580
  assumes f: "f analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   581
      and nz: "(\<And>z. z \<in> S \<Longrightarrow> f z \<noteq> 0)"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   582
    shows "(\<lambda>z. inverse (f z)) analytic_on S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   583
unfolding analytic_on_def
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   584
proof (intro ballI)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   585
  fix z
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   586
  assume z: "z \<in> S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   587
  then obtain e where e: "0 < e" and fh: "f holomorphic_on ball z e" using f
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   588
    by (metis analytic_on_def)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   589
  have "continuous_on (ball z e) f"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   590
    by (metis fh holomorphic_on_imp_continuous_on)
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   591
  then obtain e' where e': "0 < e'" and nz': "\<And>y. dist z y < e' \<Longrightarrow> f y \<noteq> 0"
66827
c94531b5007d Divided Topology_Euclidean_Space in two, creating new theory Connected. Also deleted some duplicate / variant theorems
paulson <lp15@cam.ac.uk>
parents: 66486
diff changeset
   592
    by (metis open_ball centre_in_ball continuous_on_open_avoid e z nz)
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   593
  have "(\<lambda>z. inverse (f z)) holomorphic_on ball z (min e e')"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   594
    apply (rule holomorphic_on_inverse)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   595
    apply (metis fh holomorphic_on_subset min.cobounded2 min.commute subset_ball)
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   596
    by (metis nz' mem_ball min_less_iff_conj)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   597
  then show "\<exists>e>0. (\<lambda>z. inverse (f z)) holomorphic_on ball z e"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   598
    by (metis e e' min_less_iff_conj)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   599
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   600
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   601
lemma analytic_on_divide [analytic_intros]:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   602
  assumes f: "f analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   603
      and g: "g analytic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   604
      and nz: "(\<And>z. z \<in> S \<Longrightarrow> g z \<noteq> 0)"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   605
    shows "(\<lambda>z. f z / g z) analytic_on S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   606
unfolding divide_inverse
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   607
by (metis analytic_on_inverse analytic_on_mult f g nz)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   608
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   609
lemma analytic_on_power [analytic_intros]:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   610
  "f analytic_on S \<Longrightarrow> (\<lambda>z. (f z) ^ n) analytic_on S"
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   611
by (induct n) (auto simp: analytic_on_mult)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   612
77166
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   613
lemma analytic_on_power_int [analytic_intros]:
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   614
  assumes nz: "n \<ge> 0 \<or> (\<forall>x\<in>A. f x \<noteq> 0)" and f: "f analytic_on A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   615
  shows   "(\<lambda>x. f x powi n) analytic_on A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   616
proof (cases "n \<ge> 0")
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   617
  case True
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   618
  have "(\<lambda>x. f x ^ nat n) analytic_on A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   619
    using analytic_on_power f by blast
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   620
  with True show ?thesis
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   621
    by (simp add: power_int_def)
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   622
next
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   623
  case False
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   624
  hence "(\<lambda>x. inverse (f x ^ nat (-n))) analytic_on A"
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   625
    using nz by (auto intro!: analytic_intros f)
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   626
  with False show ?thesis
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   627
    by (simp add: power_int_def power_inverse)
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   628
qed
0fb350e7477b More new material thanks to Manuel
paulson <lp15@cam.ac.uk>
parents: 75168
diff changeset
   629
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 64394
diff changeset
   630
lemma analytic_on_sum [analytic_intros]:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   631
  "(\<And>i. i \<in> I \<Longrightarrow> (f i) analytic_on S) \<Longrightarrow> (\<lambda>x. sum (\<lambda>i. f i x) I) analytic_on S"
71633
07bec530f02e cleaned proofs
nipkow
parents: 71189
diff changeset
   632
  by (induct I rule: infinite_finite_induct) (auto simp: analytic_on_add)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   633
75168
ff60b4acd6dd Added some theorems (from Wetzel)
paulson <lp15@cam.ac.uk>
parents: 74513
diff changeset
   634
lemma analytic_on_prod [analytic_intros]:
ff60b4acd6dd Added some theorems (from Wetzel)
paulson <lp15@cam.ac.uk>
parents: 74513
diff changeset
   635
  "(\<And>i. i \<in> I \<Longrightarrow> (f i) analytic_on S) \<Longrightarrow> (\<lambda>x. prod (\<lambda>i. f i x) I) analytic_on S"
ff60b4acd6dd Added some theorems (from Wetzel)
paulson <lp15@cam.ac.uk>
parents: 74513
diff changeset
   636
  by (induct I rule: infinite_finite_induct) (auto simp: analytic_on_mult)
ff60b4acd6dd Added some theorems (from Wetzel)
paulson <lp15@cam.ac.uk>
parents: 74513
diff changeset
   637
62408
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   638
lemma deriv_left_inverse:
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   639
  assumes "f holomorphic_on S" and "g holomorphic_on T"
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   640
      and "open S" and "open T"
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   641
      and "f ` S \<subseteq> T"
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   642
      and [simp]: "\<And>z. z \<in> S \<Longrightarrow> g (f z) = z"
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   643
      and "w \<in> S"
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   644
    shows "deriv f w * deriv g (f w) = 1"
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   645
proof -
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   646
  have "deriv f w * deriv g (f w) = deriv g (f w) * deriv f w"
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   647
    by (simp add: algebra_simps)
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   648
  also have "... = deriv (g o f) w"
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   649
    using assms
71189
954ee5acaae0 Split off new HOL-Complex_Analysis session from HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 71167
diff changeset
   650
    by (metis analytic_on_imp_differentiable_at analytic_on_open deriv_chain image_subset_iff)
62408
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   651
  also have "... = deriv id w"
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   652
  proof (rule complex_derivative_transform_within_open [where s=S])
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   653
    show "g \<circ> f holomorphic_on S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   654
      by (rule assms holomorphic_on_compose_gen holomorphic_intros)+
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   655
  qed (use assms in auto)
62408
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   656
  also have "... = 1"
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   657
    by simp
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   658
  finally show ?thesis .
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   659
qed
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   660
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69529
diff changeset
   661
subsection\<^marker>\<open>tag unimportant\<close>\<open>Analyticity at a point\<close>
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   662
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   663
lemma analytic_at_ball:
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   664
  "f analytic_on {z} \<longleftrightarrow> (\<exists>e. 0<e \<and> f holomorphic_on ball z e)"
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   665
  by (metis analytic_on_def singleton_iff)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   666
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   667
lemma analytic_at:
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   668
  "f analytic_on {z} \<longleftrightarrow> (\<exists>s. open s \<and> z \<in> s \<and> f holomorphic_on s)"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   669
  by (metis analytic_on_holomorphic empty_subsetI insert_subset)
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   670
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   671
lemma holomorphic_on_imp_analytic_at:
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   672
  assumes "f holomorphic_on A" "open A" "z \<in> A"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   673
  shows   "f analytic_on {z}"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   674
  using assms by (meson analytic_at)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   675
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   676
lemma analytic_on_analytic_at:
77226
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   677
  "f analytic_on s \<longleftrightarrow> (\<forall>z \<in> s. f analytic_on {z})"
69956724ad4f More material for Analysis and Complex_Analysis
paulson <lp15@cam.ac.uk>
parents: 77200
diff changeset
   678
  by (metis analytic_at_ball analytic_on_def)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   679
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   680
lemma analytic_at_two:
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   681
  "f analytic_on {z} \<and> g analytic_on {z} \<longleftrightarrow>
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   682
   (\<exists>s. open s \<and> z \<in> s \<and> f holomorphic_on s \<and> g holomorphic_on s)"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   683
  (is "?lhs = ?rhs")
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   684
proof
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   685
  assume ?lhs
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   686
  then obtain s t
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   687
    where st: "open s" "z \<in> s" "f holomorphic_on s"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   688
              "open t" "z \<in> t" "g holomorphic_on t"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   689
    by (auto simp: analytic_at)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   690
  show ?rhs
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   691
    apply (rule_tac x="s \<inter> t" in exI)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   692
    using st
69286
nipkow
parents: 69180
diff changeset
   693
    apply (auto simp: holomorphic_on_subset)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   694
    done
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   695
next
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   696
  assume ?rhs
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   697
  then show ?lhs
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   698
    by (force simp add: analytic_at)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   699
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   700
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69529
diff changeset
   701
subsection\<^marker>\<open>tag unimportant\<close>\<open>Combining theorems for derivative with ``analytic at'' hypotheses\<close>
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   702
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   703
lemma
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   704
  assumes "f analytic_on {z}" "g analytic_on {z}"
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   705
  shows complex_derivative_add_at: "deriv (\<lambda>w. f w + g w) z = deriv f z + deriv g z"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   706
    and complex_derivative_diff_at: "deriv (\<lambda>w. f w - g w) z = deriv f z - deriv g z"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   707
    and complex_derivative_mult_at: "deriv (\<lambda>w. f w * g w) z =
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   708
           f z * deriv g z + deriv f z * g z"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   709
proof -
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   710
  obtain s where s: "open s" "z \<in> s" "f holomorphic_on s" "g holomorphic_on s"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   711
    using assms by (metis analytic_at_two)
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   712
  show "deriv (\<lambda>w. f w + g w) z = deriv f z + deriv g z"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   713
    apply (rule DERIV_imp_deriv [OF DERIV_add])
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   714
    using s
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   715
    apply (auto simp: holomorphic_on_open field_differentiable_def DERIV_deriv_iff_field_differentiable)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   716
    done
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   717
  show "deriv (\<lambda>w. f w - g w) z = deriv f z - deriv g z"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   718
    apply (rule DERIV_imp_deriv [OF DERIV_diff])
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   719
    using s
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   720
    apply (auto simp: holomorphic_on_open field_differentiable_def DERIV_deriv_iff_field_differentiable)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   721
    done
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   722
  show "deriv (\<lambda>w. f w * g w) z = f z * deriv g z + deriv f z * g z"
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   723
    apply (rule DERIV_imp_deriv [OF DERIV_mult'])
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   724
    using s
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   725
    apply (auto simp: holomorphic_on_open field_differentiable_def DERIV_deriv_iff_field_differentiable)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   726
    done
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   727
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   728
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   729
lemma deriv_cmult_at:
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   730
  "f analytic_on {z} \<Longrightarrow>  deriv (\<lambda>w. c * f w) z = c * deriv f z"
71633
07bec530f02e cleaned proofs
nipkow
parents: 71189
diff changeset
   731
by (auto simp: complex_derivative_mult_at)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   732
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   733
lemma deriv_cmult_right_at:
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   734
  "f analytic_on {z} \<Longrightarrow>  deriv (\<lambda>w. f w * c) z = deriv f z * c"
71633
07bec530f02e cleaned proofs
nipkow
parents: 71189
diff changeset
   735
by (auto simp: complex_derivative_mult_at)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   736
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69529
diff changeset
   737
subsection\<^marker>\<open>tag unimportant\<close>\<open>Complex differentiation of sequences and series\<close>
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   738
61531
ab2e862263e7 Rounding function, uniform limits, cotangent, binomial identities
eberlm
parents: 61520
diff changeset
   739
(* TODO: Could probably be simplified using Uniform_Limit *)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   740
lemma has_complex_derivative_sequence:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   741
  fixes S :: "complex set"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   742
  assumes cvs: "convex S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   743
      and df:  "\<And>n x. x \<in> S \<Longrightarrow> (f n has_field_derivative f' n x) (at x within S)"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   744
      and conv: "\<And>e. 0 < e \<Longrightarrow> \<exists>N. \<forall>n x. n \<ge> N \<longrightarrow> x \<in> S \<longrightarrow> norm (f' n x - g' x) \<le> e"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   745
      and "\<exists>x l. x \<in> S \<and> ((\<lambda>n. f n x) \<longlongrightarrow> l) sequentially"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   746
    shows "\<exists>g. \<forall>x \<in> S. ((\<lambda>n. f n x) \<longlongrightarrow> g x) sequentially \<and>
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   747
                       (g has_field_derivative (g' x)) (at x within S)"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   748
proof -
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   749
  from assms obtain x l where x: "x \<in> S" and tf: "((\<lambda>n. f n x) \<longlongrightarrow> l) sequentially"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   750
    by blast
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   751
  { fix e::real assume e: "e > 0"
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   752
    then obtain N where N: "\<forall>n\<ge>N. \<forall>x. x \<in> S \<longrightarrow> cmod (f' n x - g' x) \<le> e"
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   753
      by (metis conv)
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   754
    have "\<exists>N. \<forall>n\<ge>N. \<forall>x\<in>S. \<forall>h. cmod (f' n x * h - g' x * h) \<le> e * cmod h"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   755
    proof (rule exI [of _ N], clarify)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   756
      fix n y h
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   757
      assume "N \<le> n" "y \<in> S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   758
      then have "cmod (f' n y - g' y) \<le> e"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   759
        by (metis N)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   760
      then have "cmod h * cmod (f' n y - g' y) \<le> cmod h * e"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   761
        by (auto simp: antisym_conv2 mult_le_cancel_left norm_triangle_ineq2)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   762
      then show "cmod (f' n y * h - g' y * h) \<le> e * cmod h"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   763
        by (simp add: norm_mult [symmetric] field_simps)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   764
    qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   765
  } note ** = this
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   766
  show ?thesis
68055
2cab37094fc4 more defer/prefer
paulson <lp15@cam.ac.uk>
parents: 67979
diff changeset
   767
    unfolding has_field_derivative_def
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   768
  proof (rule has_derivative_sequence [OF cvs _ _ x])
68239
0764ee22a4d1 tidy up of Derivative
paulson <lp15@cam.ac.uk>
parents: 68055
diff changeset
   769
    show "(\<lambda>n. f n x) \<longlonglongrightarrow> l"
0764ee22a4d1 tidy up of Derivative
paulson <lp15@cam.ac.uk>
parents: 68055
diff changeset
   770
      by (rule tf)
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   771
  next show "\<And>e. e > 0 \<Longrightarrow> \<forall>\<^sub>F n in sequentially. \<forall>x\<in>S. \<forall>h. cmod (f' n x * h - g' x * h) \<le> e * cmod h"
68239
0764ee22a4d1 tidy up of Derivative
paulson <lp15@cam.ac.uk>
parents: 68055
diff changeset
   772
      unfolding eventually_sequentially by (blast intro: **)
68055
2cab37094fc4 more defer/prefer
paulson <lp15@cam.ac.uk>
parents: 67979
diff changeset
   773
  qed (metis has_field_derivative_def df)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   774
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   775
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   776
lemma has_complex_derivative_series:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   777
  fixes S :: "complex set"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   778
  assumes cvs: "convex S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   779
      and df:  "\<And>n x. x \<in> S \<Longrightarrow> (f n has_field_derivative f' n x) (at x within S)"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   780
      and conv: "\<And>e. 0 < e \<Longrightarrow> \<exists>N. \<forall>n x. n \<ge> N \<longrightarrow> x \<in> S
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   781
                \<longrightarrow> cmod ((\<Sum>i<n. f' i x) - g' x) \<le> e"
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   782
      and "\<exists>x l. x \<in> S \<and> ((\<lambda>n. f n x) sums l)"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   783
    shows "\<exists>g. \<forall>x \<in> S. ((\<lambda>n. f n x) sums g x) \<and> ((g has_field_derivative g' x) (at x within S))"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   784
proof -
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   785
  from assms obtain x l where x: "x \<in> S" and sf: "((\<lambda>n. f n x) sums l)"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   786
    by blast
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   787
  { fix e::real assume e: "e > 0"
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   788
    then obtain N where N: "\<forall>n x. n \<ge> N \<longrightarrow> x \<in> S
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   789
            \<longrightarrow> cmod ((\<Sum>i<n. f' i x) - g' x) \<le> e"
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   790
      by (metis conv)
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   791
    have "\<exists>N. \<forall>n\<ge>N. \<forall>x\<in>S. \<forall>h. cmod ((\<Sum>i<n. h * f' i x) - g' x * h) \<le> e * cmod h"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   792
    proof (rule exI [of _ N], clarify)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   793
      fix n y h
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   794
      assume "N \<le> n" "y \<in> S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   795
      then have "cmod ((\<Sum>i<n. f' i y) - g' y) \<le> e"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   796
        by (metis N)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   797
      then have "cmod h * cmod ((\<Sum>i<n. f' i y) - g' y) \<le> cmod h * e"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   798
        by (auto simp: antisym_conv2 mult_le_cancel_left norm_triangle_ineq2)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   799
      then show "cmod ((\<Sum>i<n. h * f' i y) - g' y * h) \<le> e * cmod h"
64267
b9a1486e79be setsum -> sum
nipkow
parents: 63941
diff changeset
   800
        by (simp add: norm_mult [symmetric] field_simps sum_distrib_left)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   801
    qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   802
  } note ** = this
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   803
  show ?thesis
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   804
  unfolding has_field_derivative_def
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   805
  proof (rule has_derivative_series [OF cvs _ _ x])
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   806
    fix n x
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   807
    assume "x \<in> S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   808
    then show "((f n) has_derivative (\<lambda>z. z * f' n x)) (at x within S)"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   809
      by (metis df has_field_derivative_def mult_commute_abs)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   810
  next show " ((\<lambda>n. f n x) sums l)"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   811
    by (rule sf)
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   812
  next show "\<And>e. e>0 \<Longrightarrow> \<forall>\<^sub>F n in sequentially. \<forall>x\<in>S. \<forall>h. cmod ((\<Sum>i<n. h * f' i x) - g' x * h) \<le> e * cmod h"
68239
0764ee22a4d1 tidy up of Derivative
paulson <lp15@cam.ac.uk>
parents: 68055
diff changeset
   813
      unfolding eventually_sequentially by (blast intro: **)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   814
  qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   815
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   816
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 69529
diff changeset
   817
subsection\<^marker>\<open>tag unimportant\<close> \<open>Taylor on Complex Numbers\<close>
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   818
64267
b9a1486e79be setsum -> sum
nipkow
parents: 63941
diff changeset
   819
lemma sum_Suc_reindex:
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   820
  fixes f :: "nat \<Rightarrow> 'a::ab_group_add"
64267
b9a1486e79be setsum -> sum
nipkow
parents: 63941
diff changeset
   821
    shows  "sum f {0..n} = f 0 - f (Suc n) + sum (\<lambda>i. f (Suc i)) {0..n}"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   822
by (induct n) auto
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   823
69529
4ab9657b3257 capitalize proper names in lemma names
nipkow
parents: 69508
diff changeset
   824
lemma field_Taylor:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   825
  assumes S: "convex S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   826
      and f: "\<And>i x. x \<in> S \<Longrightarrow> i \<le> n \<Longrightarrow> (f i has_field_derivative f (Suc i) x) (at x within S)"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   827
      and B: "\<And>x. x \<in> S \<Longrightarrow> norm (f (Suc n) x) \<le> B"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   828
      and w: "w \<in> S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   829
      and z: "z \<in> S"
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   830
    shows "norm(f 0 z - (\<Sum>i\<le>n. f i w * (z-w) ^ i / (fact i)))
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   831
          \<le> B * norm(z - w)^(Suc n) / fact n"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   832
proof -
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   833
  have wzs: "closed_segment w z \<subseteq> S" using assms
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   834
    by (metis convex_contains_segment)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   835
  { fix u
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   836
    assume "u \<in> closed_segment w z"
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   837
    then have "u \<in> S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   838
      by (metis wzs subsetD)
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   839
    have "(\<Sum>i\<le>n. f i u * (- of_nat i * (z-u)^(i - 1)) / (fact i) +
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   840
                      f (Suc i) u * (z-u)^i / (fact i)) =
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   841
              f (Suc n) u * (z-u) ^ n / (fact n)"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   842
    proof (induction n)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   843
      case 0 show ?case by simp
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   844
    next
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   845
      case (Suc n)
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   846
      have "(\<Sum>i\<le>Suc n. f i u * (- of_nat i * (z-u) ^ (i - 1)) / (fact i) +
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   847
                             f (Suc i) u * (z-u) ^ i / (fact i)) =
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   848
           f (Suc n) u * (z-u) ^ n / (fact n) +
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   849
           f (Suc (Suc n)) u * ((z-u) * (z-u) ^ n) / (fact (Suc n)) -
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   850
           f (Suc n) u * ((1 + of_nat n) * (z-u) ^ n) / (fact (Suc n))"
56479
91958d4b30f7 revert c1bbd3e22226, a14831ac3023, and 36489d77c484: divide_minus_left/right are again simp rules
hoelzl
parents: 56409
diff changeset
   851
        using Suc by simp
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   852
      also have "... = f (Suc (Suc n)) u * (z-u) ^ Suc n / (fact (Suc n))"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   853
      proof -
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   854
        have "(fact(Suc n)) *
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   855
             (f(Suc n) u *(z-u) ^ n / (fact n) +
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   856
               f(Suc(Suc n)) u *((z-u) *(z-u) ^ n) / (fact(Suc n)) -
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   857
               f(Suc n) u *((1 + of_nat n) *(z-u) ^ n) / (fact(Suc n))) =
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   858
            ((fact(Suc n)) *(f(Suc n) u *(z-u) ^ n)) / (fact n) +
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   859
            ((fact(Suc n)) *(f(Suc(Suc n)) u *((z-u) *(z-u) ^ n)) / (fact(Suc n))) -
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   860
            ((fact(Suc n)) *(f(Suc n) u *(of_nat(Suc n) *(z-u) ^ n))) / (fact(Suc n))"
63367
6c731c8b7f03 simplified definitions of combinatorial functions
haftmann
parents: 63332
diff changeset
   861
          by (simp add: algebra_simps del: fact_Suc)
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   862
        also have "... = ((fact (Suc n)) * (f (Suc n) u * (z-u) ^ n)) / (fact n) +
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   863
                         (f (Suc (Suc n)) u * ((z-u) * (z-u) ^ n)) -
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   864
                         (f (Suc n) u * ((1 + of_nat n) * (z-u) ^ n))"
63367
6c731c8b7f03 simplified definitions of combinatorial functions
haftmann
parents: 63332
diff changeset
   865
          by (simp del: fact_Suc)
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   866
        also have "... = (of_nat (Suc n) * (f (Suc n) u * (z-u) ^ n)) +
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   867
                         (f (Suc (Suc n)) u * ((z-u) * (z-u) ^ n)) -
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   868
                         (f (Suc n) u * ((1 + of_nat n) * (z-u) ^ n))"
63367
6c731c8b7f03 simplified definitions of combinatorial functions
haftmann
parents: 63332
diff changeset
   869
          by (simp only: fact_Suc of_nat_mult ac_simps) simp
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   870
        also have "... = f (Suc (Suc n)) u * ((z-u) * (z-u) ^ n)"
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   871
          by (simp add: algebra_simps)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   872
        finally show ?thesis
63367
6c731c8b7f03 simplified definitions of combinatorial functions
haftmann
parents: 63332
diff changeset
   873
        by (simp add: mult_left_cancel [where c = "(fact (Suc n))", THEN iffD1] del: fact_Suc)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   874
      qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   875
      finally show ?case .
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   876
    qed
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   877
    then have "((\<lambda>v. (\<Sum>i\<le>n. f i v * (z - v)^i / (fact i)))
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   878
                has_field_derivative f (Suc n) u * (z-u) ^ n / (fact n))
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   879
               (at u within S)"
56381
0556204bc230 merged DERIV_intros, has_derivative_intros into derivative_intros
hoelzl
parents: 56371
diff changeset
   880
      apply (intro derivative_eq_intros)
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   881
      apply (blast intro: assms \<open>u \<in> S\<close>)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   882
      apply (rule refl)+
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   883
      apply (auto simp: field_simps)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   884
      done
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   885
  } note sum_deriv = this
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   886
  { fix u
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   887
    assume u: "u \<in> closed_segment w z"
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   888
    then have us: "u \<in> S"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   889
      by (metis wzs subsetD)
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   890
    have "norm (f (Suc n) u) * norm (z - u) ^ n \<le> norm (f (Suc n) u) * norm (u - z) ^ n"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   891
      by (metis norm_minus_commute order_refl)
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   892
    also have "... \<le> norm (f (Suc n) u) * norm (z - w) ^ n"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   893
      by (metis mult_left_mono norm_ge_zero power_mono segment_bound [OF u])
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   894
    also have "... \<le> B * norm (z - w) ^ n"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   895
      by (metis norm_ge_zero zero_le_power mult_right_mono  B [OF us])
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   896
    finally have "norm (f (Suc n) u) * norm (z - u) ^ n \<le> B * norm (z - w) ^ n" .
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   897
  } note cmod_bound = this
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   898
  have "(\<Sum>i\<le>n. f i z * (z - z) ^ i / (fact i)) = (\<Sum>i\<le>n. (f i z / (fact i)) * 0 ^ i)"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   899
    by simp
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   900
  also have "\<dots> = f 0 z / (fact 0)"
64267
b9a1486e79be setsum -> sum
nipkow
parents: 63941
diff changeset
   901
    by (subst sum_zero_power) simp
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   902
  finally have "norm (f 0 z - (\<Sum>i\<le>n. f i w * (z - w) ^ i / (fact i)))
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   903
                \<le> norm ((\<Sum>i\<le>n. f i w * (z - w) ^ i / (fact i)) -
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   904
                        (\<Sum>i\<le>n. f i z * (z - z) ^ i / (fact i)))"
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   905
    by (simp add: norm_minus_commute)
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   906
  also have "... \<le> B * norm (z - w) ^ n / (fact n) * norm (w - z)"
62534
6855b348e828 complex_differentiable -> field_differentiable, etc. (making these theorems also available for type real)
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
   907
    apply (rule field_differentiable_bound
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   908
      [where f' = "\<lambda>w. f (Suc n) w * (z - w)^n / (fact n)"
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   909
         and S = "closed_segment w z", OF convex_closed_segment])
71633
07bec530f02e cleaned proofs
nipkow
parents: 71189
diff changeset
   910
    apply (auto simp: DERIV_subset [OF sum_deriv wzs]
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   911
                  norm_divide norm_mult norm_power divide_le_cancel cmod_bound)
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   912
    done
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   913
  also have "...  \<le> B * norm (z - w) ^ Suc n / (fact n)"
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   914
    by (simp add: algebra_simps norm_minus_commute)
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   915
  finally show ?thesis .
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   916
qed
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
   917
69529
4ab9657b3257 capitalize proper names in lemma names
nipkow
parents: 69508
diff changeset
   918
lemma complex_Taylor:
68255
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   919
  assumes S: "convex S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   920
      and f: "\<And>i x. x \<in> S \<Longrightarrow> i \<le> n \<Longrightarrow> (f i has_field_derivative f (Suc i) x) (at x within S)"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   921
      and B: "\<And>x. x \<in> S \<Longrightarrow> cmod (f (Suc n) x) \<le> B"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   922
      and w: "w \<in> S"
009f783d1bac small clean-up of Complex_Analysis_Basics
paulson <lp15@cam.ac.uk>
parents: 68239
diff changeset
   923
      and z: "z \<in> S"
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   924
    shows "cmod(f 0 z - (\<Sum>i\<le>n. f i w * (z-w) ^ i / (fact i)))
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   925
          \<le> B * cmod(z - w)^(Suc n) / fact n"
69529
4ab9657b3257 capitalize proper names in lemma names
nipkow
parents: 69508
diff changeset
   926
  using assms by (rule field_Taylor)
66252
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   927
b73f94b366b7 some generalizations complex=>real_normed_field
immler
parents: 66089
diff changeset
   928
62408
86f27b264d3d Conformal_mappings: a big development in complex analysis (+ some lemmas)
paulson <lp15@cam.ac.uk>
parents: 62397
diff changeset
   929
text\<open>Something more like the traditional MVT for real components\<close>
56370
7c717ba55a0b reorder Complex_Analysis_Basics; rename DD to deriv
hoelzl
parents: 56369
diff changeset
   930
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   931
lemma complex_mvt_line:
56369
2704ca85be98 moved generic theorems from Complex_Analysis_Basic; fixed some theorem names
hoelzl
parents: 56332
diff changeset
   932
  assumes "\<And>u. u \<in> closed_segment w z \<Longrightarrow> (f has_field_derivative f'(u)) (at u)"
61518
ff12606337e9 new lemmas about topology, etc., for Cauchy integral formula
paulson
parents: 61235
diff changeset
   933
    shows "\<exists>u. u \<in> closed_segment w z \<and> Re(f z) - Re(f w) = Re(f'(u) * (z - w))"
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   934
proof -
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   935
  have twz: "\<And>t. (1 - t) *\<^sub>R w + t *\<^sub>R z = w + t *\<^sub>R (z - w)"
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   936
    by (simp add: real_vector.scale_left_diff_distrib real_vector.scale_right_diff_distrib)
56381
0556204bc230 merged DERIV_intros, has_derivative_intros into derivative_intros
hoelzl
parents: 56371
diff changeset
   937
  note assms[unfolded has_field_derivative_def, derivative_intros]
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   938
  show ?thesis
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   939
    apply (cut_tac mvt_simple
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   940
                     [of 0 1 "Re o f o (\<lambda>t. (1 - t) *\<^sub>R w +  t *\<^sub>R z)"
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   941
                      "\<lambda>u. Re o (\<lambda>h. f'((1 - u) *\<^sub>R w + u *\<^sub>R z) * h) o (\<lambda>t. t *\<^sub>R (z - w))"])
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   942
    apply auto
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   943
    apply (rule_tac x="(1 - x) *\<^sub>R w + x *\<^sub>R z" in exI)
61518
ff12606337e9 new lemmas about topology, etc., for Cauchy integral formula
paulson
parents: 61235
diff changeset
   944
    apply (auto simp: closed_segment_def twz) []
67979
53323937ee25 new material about vec, real^1, etc.
paulson <lp15@cam.ac.uk>
parents: 67968
diff changeset
   945
    apply (intro derivative_eq_intros has_derivative_at_withinI, simp_all)
56369
2704ca85be98 moved generic theorems from Complex_Analysis_Basic; fixed some theorem names
hoelzl
parents: 56332
diff changeset
   946
    apply (simp add: fun_eq_iff real_vector.scale_right_diff_distrib)
61518
ff12606337e9 new lemmas about topology, etc., for Cauchy integral formula
paulson
parents: 61235
diff changeset
   947
    apply (force simp: twz closed_segment_def)
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   948
    done
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   949
qed
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   950
69529
4ab9657b3257 capitalize proper names in lemma names
nipkow
parents: 69508
diff changeset
   951
lemma complex_Taylor_mvt:
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   952
  assumes "\<And>i x. \<lbrakk>x \<in> closed_segment w z; i \<le> n\<rbrakk> \<Longrightarrow> ((f i) has_field_derivative f (Suc i) x) (at x)"
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   953
    shows "\<exists>u. u \<in> closed_segment w z \<and>
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   954
            Re (f 0 z) =
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   955
            Re ((\<Sum>i = 0..n. f i w * (z - w) ^ i / (fact i)) +
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   956
                (f (Suc n) u * (z-u)^n / (fact n)) * (z - w))"
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   957
proof -
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   958
  { fix u
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   959
    assume u: "u \<in> closed_segment w z"
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   960
    have "(\<Sum>i = 0..n.
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   961
               (f (Suc i) u * (z-u) ^ i - of_nat i * (f i u * (z-u) ^ (i - Suc 0))) /
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   962
               (fact i)) =
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   963
          f (Suc 0) u -
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   964
             (f (Suc (Suc n)) u * ((z-u) ^ Suc n) - (of_nat (Suc n)) * (z-u) ^ n * f (Suc n) u) /
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   965
             (fact (Suc n)) +
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   966
             (\<Sum>i = 0..n.
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   967
                 (f (Suc (Suc i)) u * ((z-u) ^ Suc i) - of_nat (Suc i) * (f (Suc i) u * (z-u) ^ i)) /
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   968
                 (fact (Suc i)))"
64267
b9a1486e79be setsum -> sum
nipkow
parents: 63941
diff changeset
   969
       by (subst sum_Suc_reindex) simp
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   970
    also have "... = f (Suc 0) u -
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   971
             (f (Suc (Suc n)) u * ((z-u) ^ Suc n) - (of_nat (Suc n)) * (z-u) ^ n * f (Suc n) u) /
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   972
             (fact (Suc n)) +
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   973
             (\<Sum>i = 0..n.
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   974
                 f (Suc (Suc i)) u * ((z-u) ^ Suc i) / (fact (Suc i))  -
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   975
                 f (Suc i) u * (z-u) ^ i / (fact i))"
57514
bdc2c6b40bf2 prefer ac_simps collections over separate name bindings for add and mult
haftmann
parents: 56889
diff changeset
   976
      by (simp only: diff_divide_distrib fact_cancel ac_simps)
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   977
    also have "... = f (Suc 0) u -
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   978
             (f (Suc (Suc n)) u * (z-u) ^ Suc n - of_nat (Suc n) * (z-u) ^ n * f (Suc n) u) /
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   979
             (fact (Suc n)) +
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   980
             f (Suc (Suc n)) u * (z-u) ^ Suc n / (fact (Suc n)) - f (Suc 0) u"
64267
b9a1486e79be setsum -> sum
nipkow
parents: 63941
diff changeset
   981
      by (subst sum_Suc_diff) auto
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   982
    also have "... = f (Suc n) u * (z-u) ^ n / (fact n)"
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   983
      by (simp only: algebra_simps diff_divide_distrib fact_cancel)
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61531
diff changeset
   984
    finally have "(\<Sum>i = 0..n. (f (Suc i) u * (z - u) ^ i
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   985
                             - of_nat i * (f i u * (z-u) ^ (i - Suc 0))) / (fact i)) =
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   986
                  f (Suc n) u * (z - u) ^ n / (fact n)" .
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   987
    then have "((\<lambda>u. \<Sum>i = 0..n. f i u * (z - u) ^ i / (fact i)) has_field_derivative
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   988
                f (Suc n) u * (z - u) ^ n / (fact n))  (at u)"
56381
0556204bc230 merged DERIV_intros, has_derivative_intros into derivative_intros
hoelzl
parents: 56371
diff changeset
   989
      apply (intro derivative_eq_intros)+
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   990
      apply (force intro: u assms)
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   991
      apply (rule refl)+
57514
bdc2c6b40bf2 prefer ac_simps collections over separate name bindings for add and mult
haftmann
parents: 56889
diff changeset
   992
      apply (auto simp: ac_simps)
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   993
      done
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   994
  }
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   995
  then show ?thesis
59730
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   996
    apply (cut_tac complex_mvt_line [of w z "\<lambda>u. \<Sum>i = 0..n. f i u * (z-u) ^ i / (fact i)"
b7c394c7a619 The factorial function, "fact", now has type "nat => 'a"
paulson <lp15@cam.ac.uk>
parents: 59615
diff changeset
   997
               "\<lambda>u. (f (Suc n) u * (z-u)^n / (fact n))"])
56238
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   998
    apply (auto simp add: intro: open_closed_segment)
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
   999
    done
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
  1000
qed
5d147e1e18d1 a few new lemmas and generalisations of old ones
paulson <lp15@cam.ac.uk>
parents: 56223
diff changeset
  1001
60017
b785d6d06430 Overloading of ln and powr, but "approximation" no longer works for powr. Code generation also fails due to type ambiguity in scala.
paulson <lp15@cam.ac.uk>
parents: 59730
diff changeset
  1002
56215
fcf90317383d New complex analysis material
paulson <lp15@cam.ac.uk>
parents:
diff changeset
  1003
end