src/HOL/Probability/Regularity.thy
changeset 59452 2538b2c51769
parent 58876 1888e3cb8048
child 60017 b785d6d06430
--- a/src/HOL/Probability/Regularity.thy	Mon Jan 26 14:40:13 2015 +0100
+++ b/src/HOL/Probability/Regularity.thy	Tue Jan 27 16:12:40 2015 +0100
@@ -312,7 +312,7 @@
     case 2
     have "M (space M - B) = M (space M) - emeasure M B" by (auto simp: emeasure_compl)
     also have "\<dots> = (INF K:{K. K \<subseteq> B \<and> compact K}. M (space M) -  M K)"
-      unfolding inner by (subst INF_ereal_cminus) force+
+      unfolding inner by (subst INF_ereal_minus_right) force+
     also have "\<dots> = (INF U:{U. U \<subseteq> B \<and> compact U}. M (space M - U))"
       by (rule INF_cong) (auto simp add: emeasure_compl sb compact_imp_closed)
     also have "\<dots> \<ge> (INF U:{U. U \<subseteq> B \<and> closed U}. M (space M - U))"
@@ -331,7 +331,7 @@
     case 1
     have "M (space M - B) = M (space M) - emeasure M B" by (auto simp: emeasure_compl)
     also have "\<dots> = (SUP U: {U. B \<subseteq> U \<and> open U}. M (space M) -  M U)"
-      unfolding outer by (subst SUP_ereal_cminus) auto
+      unfolding outer by (subst SUP_ereal_minus_right) auto
     also have "\<dots> = (SUP U:{U. B \<subseteq> U \<and> open U}. M (space M - U))"
       by (rule SUP_cong) (auto simp add: emeasure_compl sb compact_imp_closed)
     also have "\<dots> = (SUP K:{K. K \<subseteq> space M - B \<and> closed K}. emeasure M K)"