src/HOL/Probability/Borel_Space.thy
changeset 46884 154dc6ec0041
parent 46731 5302e932d1e5
child 46905 6b1c0a80a57a
--- a/src/HOL/Probability/Borel_Space.thy	Mon Mar 12 15:12:22 2012 +0100
+++ b/src/HOL/Probability/Borel_Space.thy	Mon Mar 12 21:41:11 2012 +0100
@@ -1417,7 +1417,7 @@
 proof
   fix a
   have "?sup -` {a<..} \<inter> space M = (\<Union>i\<in>A. {x\<in>space M. a < f i x})"
-    by (auto simp: less_SUP_iff SUP_apply)
+    by (auto simp: less_SUP_iff)
   then show "?sup -` {a<..} \<inter> space M \<in> sets M"
     using assms by auto
 qed
@@ -1430,7 +1430,7 @@
 proof
   fix a
   have "?inf -` {..<a} \<inter> space M = (\<Union>i\<in>A. {x\<in>space M. f i x < a})"
-    by (auto simp: INF_less_iff INF_apply)
+    by (auto simp: INF_less_iff)
   then show "?inf -` {..<a} \<inter> space M \<in> sets M"
     using assms by auto
 qed