diff -r 261d42f0bfac -r 979cdfdf7a79 src/HOL/Probability/Levy.thy --- a/src/HOL/Probability/Levy.thy Mon Oct 17 15:20:06 2016 +0200 +++ b/src/HOL/Probability/Levy.thy Thu Oct 13 18:36:06 2016 +0200 @@ -390,7 +390,7 @@ by (intro borel_integrable_compact[OF compact_Icc] continuous_at_imp_continuous_on continuous_intros ballI M'.isCont_char continuous_intros) have "cmod (CLBINT t:{-d/2..d/2}. 1 - char M' t) \ LBINT t:{-d/2..d/2}. cmod (1 - char M' t)" - using integral_norm_bound[OF 2] by simp + using integral_norm_bound[of _ "\x. indicator {u..v} x *\<^sub>R (1 - char M' x)" for u v] by simp also have 4: "\ \ LBINT t:{-d/2..d/2}. \ / 4" apply (rule integral_mono [OF 3]) apply (simp add: emeasure_lborel_Icc_eq)