src/HOL/Probability/Giry_Monad.thy
changeset 63092 a949b2a5f51d
parent 63040 eb4ddd18d635
child 63333 158ab2239496
equal deleted inserted replaced
63091:54f16a0a3069 63092:a949b2a5f51d
   769     apply (auto simp: space_subprob_algebra
   769     apply (auto simp: space_subprob_algebra
   770                  dest!: sets_eq_imp_space_eq subprob_space.emeasure_space_le_1)
   770                  dest!: sets_eq_imp_space_eq subprob_space.emeasure_space_le_1)
   771     done
   771     done
   772   with M show "subprob_space (join M)"
   772   with M show "subprob_space (join M)"
   773     by (intro subprob_spaceI)
   773     by (intro subprob_spaceI)
   774        (auto simp: emeasure_join space_subprob_algebra M assms dest: subprob_space.emeasure_space_le_1)
   774        (auto simp: emeasure_join space_subprob_algebra M dest: subprob_space.emeasure_space_le_1)
   775 next
   775 next
   776   assume "\<not>(space N \<noteq> {})"
   776   assume "\<not>(space N \<noteq> {})"
   777   thus ?thesis by (simp add: measurable_empty_iff space_subprob_algebra_empty_iff)
   777   thus ?thesis by (simp add: measurable_empty_iff space_subprob_algebra_empty_iff)
   778 qed (auto simp: space_subprob_algebra)
   778 qed (auto simp: space_subprob_algebra)
   779 
   779