src/HOL/Probability/Lebesgue_Integration.thy
changeset 46884 154dc6ec0041
parent 46731 5302e932d1e5
child 46905 6b1c0a80a57a
--- a/src/HOL/Probability/Lebesgue_Integration.thy	Mon Mar 12 15:12:22 2012 +0100
+++ b/src/HOL/Probability/Lebesgue_Integration.thy	Mon Mar 12 21:41:11 2012 +0100
@@ -1044,7 +1044,7 @@
         with `a < 1` u_range[OF `x \<in> space M`]
         have "a * u x < 1 * u x"
           by (intro ereal_mult_strict_right_mono) (auto simp: image_iff)
-        also have "\<dots> \<le> (SUP i. f i x)" using u(2) by (auto simp: le_fun_def SUP_apply)
+        also have "\<dots> \<le> (SUP i. f i x)" using u(2) by (auto simp: le_fun_def)
         finally obtain i where "a * u x < f i x" unfolding SUP_def
           by (auto simp add: less_Sup_iff)
         hence "a * u x \<le> f i x" by auto
@@ -1115,7 +1115,7 @@
       using f by (auto intro!: SUP_upper2)
     ultimately show "integral\<^isup>S M g \<le> (SUP j. integral\<^isup>P M (f j))"
       by (intro  positive_integral_SUP_approx[OF f g _ g'])
-         (auto simp: le_fun_def max_def SUP_apply)
+         (auto simp: le_fun_def max_def)
   qed
 qed