src/HOL/Multivariate_Analysis/Cauchy_Integral_Thm.thy
changeset 63262 e497387de7af
parent 63092 a949b2a5f51d
child 63367 6c731c8b7f03
--- a/src/HOL/Multivariate_Analysis/Cauchy_Integral_Thm.thy	Wed Jun 08 19:36:45 2016 +0200
+++ b/src/HOL/Multivariate_Analysis/Cauchy_Integral_Thm.thy	Thu Jun 09 16:11:33 2016 +0200
@@ -6289,13 +6289,13 @@
   obtain B where B: "\<And>x. B \<le> cmod x \<Longrightarrow> norm (f x) * 2 < cmod (f z)"
     by (auto simp: dist_norm)
   define R where "R = 1 + \<bar>B\<bar> + norm z"
-  have "R > 0" unfolding R_def 
+  have "R > 0" unfolding R_def
   proof -
     have "0 \<le> cmod z + \<bar>B\<bar>"
       by (metis (full_types) add_nonneg_nonneg norm_ge_zero real_norm_def)
     then show "0 < 1 + \<bar>B\<bar> + cmod z"
       by linarith
-  qed 
+  qed
   have *: "((\<lambda>u. f u / (u - z)) has_contour_integral 2 * complex_of_real pi * \<i> * f z) (circlepath z R)"
     apply (rule Cauchy_integral_circlepath)
     using \<open>R > 0\<close> apply (auto intro: holomorphic_on_subset [OF holf] holomorphic_on_imp_continuous_on)+