src/HOL/Probability/Caratheodory.thy
changeset 51329 4a3c453f99a1
parent 49773 16907431e477
child 52141 eff000cab70f
equal deleted inserted replaced
51328:d63ec23c9125 51329:4a3c453f99a1
   361 
   361 
   362 lemma (in ring_of_sets) inf_measure_agrees:
   362 lemma (in ring_of_sets) inf_measure_agrees:
   363   assumes posf: "positive M f" and ca: "countably_additive M f"
   363   assumes posf: "positive M f" and ca: "countably_additive M f"
   364       and s: "s \<in> M"
   364       and s: "s \<in> M"
   365   shows "Inf (measure_set M f s) = f s"
   365   shows "Inf (measure_set M f s) = f s"
   366   unfolding Inf_ereal_def
   366 proof (intro Inf_eqI)
   367 proof (safe intro!: Greatest_equality)
       
   368   fix z
   367   fix z
   369   assume z: "z \<in> measure_set M f s"
   368   assume z: "z \<in> measure_set M f s"
   370   from this obtain A where
   369   from this obtain A where
   371     A: "range A \<subseteq> M" and disj: "disjoint_family A"
   370     A: "range A \<subseteq> M" and disj: "disjoint_family A"
   372     and "s \<subseteq> (\<Union>x. A x)" and si: "(\<Sum>i. f (A i)) = z"
   371     and "s \<subseteq> (\<Union>x. A x)" and si: "(\<Sum>i. f (A i)) = z"
   392       fix N have "A N \<inter> s \<in> M"  using A s by auto
   391       fix N have "A N \<inter> s \<in> M"  using A s by auto
   393       then show "0 \<le> f (A N \<inter> s)" using posf unfolding positive_def by auto
   392       then show "0 \<le> f (A N \<inter> s)" using posf unfolding positive_def by auto
   394     qed
   393     qed
   395   also have "... = z" by (rule si)
   394   also have "... = z" by (rule si)
   396   finally show "f s \<le> z" .
   395   finally show "f s \<le> z" .
   397 next
   396 qed (blast intro: inf_measure_nonempty [of _ f, OF posf s subset_refl])
   398   fix y
       
   399   assume y: "\<forall>u \<in> measure_set M f s. y \<le> u"
       
   400   thus "y \<le> f s"
       
   401     by (blast intro: inf_measure_nonempty [of _ f, OF posf s subset_refl])
       
   402 qed
       
   403 
   397 
   404 lemma measure_set_pos:
   398 lemma measure_set_pos:
   405   assumes posf: "positive M f" "r \<in> measure_set M f X"
   399   assumes posf: "positive M f" "r \<in> measure_set M f X"
   406   shows "0 \<le> r"
   400   shows "0 \<le> r"
   407 proof -
   401 proof -