src/HOL/Analysis/Cauchy_Integral_Theorem.thy
changeset 63928 d81fb5b46a5c
parent 63918 6bf55e6e0b75
child 63938 f6ce08859d4c
equal deleted inserted replaced
63927:0efb482beb84 63928:d81fb5b46a5c
  5418 by (auto simp: vector_derivative_circlepath norm_mult intro: contour_integral_uniform_limit assms)
  5418 by (auto simp: vector_derivative_circlepath norm_mult intro: contour_integral_uniform_limit assms)
  5419 
  5419 
  5420 
  5420 
  5421 subsection\<open> General stepping result for derivative formulas.\<close>
  5421 subsection\<open> General stepping result for derivative formulas.\<close>
  5422 
  5422 
  5423 lemma sum_sqs_eq:
       
  5424   fixes x::"'a::idom" shows "x * x + y * y = x * (y * 2) \<Longrightarrow> y = x"
       
  5425   by algebra
       
  5426 
       
  5427 proposition Cauchy_next_derivative:
  5423 proposition Cauchy_next_derivative:
  5428   assumes "continuous_on (path_image \<gamma>) f'"
  5424   assumes "continuous_on (path_image \<gamma>) f'"
  5429       and leB: "\<And>t. t \<in> {0..1} \<Longrightarrow> norm (vector_derivative \<gamma> (at t)) \<le> B"
  5425       and leB: "\<And>t. t \<in> {0..1} \<Longrightarrow> norm (vector_derivative \<gamma> (at t)) \<le> B"
  5430       and int: "\<And>w. w \<in> s - path_image \<gamma> \<Longrightarrow> ((\<lambda>u. f' u / (u - w)^k) has_contour_integral f w) \<gamma>"
  5426       and int: "\<And>w. w \<in> s - path_image \<gamma> \<Longrightarrow> ((\<lambda>u. f' u / (u - w)^k) has_contour_integral f w) \<gamma>"
  5431       and k: "k \<noteq> 0"
  5427       and k: "k \<noteq> 0"