src/HOL/Probability/Lebesgue_Integral_Substitution.thy
changeset 59452 2538b2c51769
parent 59092 d469103c0737
child 61609 77b453bd616f
--- a/src/HOL/Probability/Lebesgue_Integral_Substitution.thy	Mon Jan 26 14:40:13 2015 +0100
+++ b/src/HOL/Probability/Lebesgue_Integral_Substitution.thy	Tue Jan 27 16:12:40 2015 +0100
@@ -566,7 +566,7 @@
          (auto simp: incseq_def le_fun_def derivg_nonneg Mf' split: split_indicator
                intro!: ereal_mult_right_mono)
     also from sup have "... = \<integral>\<^sup>+x. (SUP i. F i (g x)) * ereal (g' x) * indicator {a..b} x \<partial>lborel"
-      by (subst mult.assoc, subst mult.commute, subst SUP_ereal_cmult)
+      by (subst mult.assoc, subst mult.commute, subst SUP_ereal_mult_left)
          (auto split: split_indicator simp: derivg_nonneg mult_ac)
     finally show ?case by simp
   qed