src/HOL/Probability/Caratheodory.thy
changeset 51329 4a3c453f99a1
parent 49773 16907431e477
child 52141 eff000cab70f
--- a/src/HOL/Probability/Caratheodory.thy	Wed Feb 20 12:04:42 2013 +0100
+++ b/src/HOL/Probability/Caratheodory.thy	Wed Feb 20 12:04:42 2013 +0100
@@ -363,8 +363,7 @@
   assumes posf: "positive M f" and ca: "countably_additive M f"
       and s: "s \<in> M"
   shows "Inf (measure_set M f s) = f s"
-  unfolding Inf_ereal_def
-proof (safe intro!: Greatest_equality)
+proof (intro Inf_eqI)
   fix z
   assume z: "z \<in> measure_set M f s"
   from this obtain A where
@@ -394,12 +393,7 @@
     qed
   also have "... = z" by (rule si)
   finally show "f s \<le> z" .
-next
-  fix y
-  assume y: "\<forall>u \<in> measure_set M f s. y \<le> u"
-  thus "y \<le> f s"
-    by (blast intro: inf_measure_nonempty [of _ f, OF posf s subset_refl])
-qed
+qed (blast intro: inf_measure_nonempty [of _ f, OF posf s subset_refl])
 
 lemma measure_set_pos:
   assumes posf: "positive M f" "r \<in> measure_set M f X"