src/HOL/Complex_Analysis/Contour_Integration.thy
changeset 82400 24d09a911713
parent 81874 067462a6a652
child 82517 111b1b2a2d13
--- a/src/HOL/Complex_Analysis/Contour_Integration.thy	Thu Apr 03 21:08:36 2025 +0100
+++ b/src/HOL/Complex_Analysis/Contour_Integration.thy	Fri Apr 04 16:37:58 2025 +0100
@@ -808,7 +808,7 @@
           "0 \<le> B" and B: "\<And>x. x \<in> closed_segment a b \<Longrightarrow> norm(f x) \<le> B"
     shows "norm i \<le> B * norm(b - a)"
 proof -
-  have "norm i \<le> (B * norm (b - a)) * content (cbox 0 (1::real))"
+  have "norm i \<le> (B * norm (b - a)) * measure lborel (cbox 0 (1::real))"
   proof (rule has_integral_bound
        [of _ "\<lambda>x. f (linepath a b x) * vector_derivative (linepath a b) (at x within {0..1})"])
     show  "cmod (f (linepath a b x) * vector_derivative (linepath a b) (at x within {0..1}))