src/HOL/Multivariate_Analysis/Cauchy_Integral_Thm.thy
changeset 62533 bc25f3916a99
parent 62464 08e62096e7f4
child 62534 6855b348e828
equal deleted inserted replaced
62532:edee1966fddf 62533:bc25f3916a99
  2676 qed
  2676 qed
  2677 
  2677 
  2678 (** Existence of a primitive.*)
  2678 (** Existence of a primitive.*)
  2679 
  2679 
  2680 lemma holomorphic_starlike_primitive:
  2680 lemma holomorphic_starlike_primitive:
       
  2681   fixes f :: "complex \<Rightarrow> complex"
  2681   assumes contf: "continuous_on s f"
  2682   assumes contf: "continuous_on s f"
  2682       and s: "starlike s" and os: "open s"
  2683       and s: "starlike s" and os: "open s"
  2683       and k: "finite k"
  2684       and k: "finite k"
  2684       and fcd: "\<And>x. x \<in> s - k \<Longrightarrow> f complex_differentiable at x"
  2685       and fcd: "\<And>x. x \<in> s - k \<Longrightarrow> f complex_differentiable at x"
  2685     shows "\<exists>g. \<forall>x \<in> s. (g has_field_derivative f x) (at x)"
  2686     shows "\<exists>g. \<forall>x \<in> s. (g has_field_derivative f x) (at x)"
  2794   apply (simp_all add: ex_in_conv [symmetric])
  2795   apply (simp_all add: ex_in_conv [symmetric])
  2795   apply (blast intro: triangle_contour_integrals_convex_primitive has_chain_integral_chain_integral3)
  2796   apply (blast intro: triangle_contour_integrals_convex_primitive has_chain_integral_chain_integral3)
  2796   done
  2797   done
  2797 
  2798 
  2798 lemma holomorphic_convex_primitive:
  2799 lemma holomorphic_convex_primitive:
       
  2800   fixes f :: "complex \<Rightarrow> complex"
       
  2801   shows
  2799   "\<lbrakk>convex s; finite k; continuous_on s f;
  2802   "\<lbrakk>convex s; finite k; continuous_on s f;
  2800     \<And>x. x \<in> interior s - k \<Longrightarrow> f complex_differentiable at x\<rbrakk>
  2803     \<And>x. x \<in> interior s - k \<Longrightarrow> f complex_differentiable at x\<rbrakk>
  2801    \<Longrightarrow> \<exists>g. \<forall>x \<in> s. (g has_field_derivative f x) (at x within s)"
  2804    \<Longrightarrow> \<exists>g. \<forall>x \<in> s. (g has_field_derivative f x) (at x within s)"
  2802 apply (rule contour_integral_convex_primitive [OF _ _ Cauchy_theorem_triangle_cofinite])
  2805 apply (rule contour_integral_convex_primitive [OF _ _ Cauchy_theorem_triangle_cofinite])
  2803 prefer 3
  2806 prefer 3