diff -r 85ed00c1fe7c -r 340738057c8c src/HOL/Probability/Bochner_Integration.thy --- a/src/HOL/Probability/Bochner_Integration.thy Fri Feb 19 13:40:50 2016 +0100 +++ b/src/HOL/Probability/Bochner_Integration.thy Mon Feb 22 14:37:56 2016 +0000 @@ -1229,7 +1229,7 @@ s: "\i. simple_function M (s i)" and pointwise: "\x. x \ space M \ (\i. s i x) \ f x" and bound: "\i x. x \ space M \ norm (s i x) \ 2 * norm (f x)" - by (simp add: norm_conv_dist) metis + by simp metis show ?thesis proof (rule integrableI_sequence) @@ -2545,7 +2545,7 @@ then have s: "\i. simple_function (N \\<^sub>M M) (s i)" "\x y. x \ space N \ y \ space M \ (\i. s i (x, y)) \ f x y" "\i x y. x \ space N \ y \ space M \ norm (s i (x, y)) \ 2 * norm (f x y)" - by (auto simp: space_pair_measure norm_conv_dist) + by (auto simp: space_pair_measure) have [measurable]: "\i. s i \ borel_measurable (N \\<^sub>M M)" by (rule borel_measurable_simple_function) fact