src/HOL/Probability/Binary_Product_Measure.thy
changeset 59000 6eb0725503fc
parent 58876 1888e3cb8048
child 59048 7dc8ac6f0895
--- a/src/HOL/Probability/Binary_Product_Measure.thy	Thu Nov 13 14:40:06 2014 +0100
+++ b/src/HOL/Probability/Binary_Product_Measure.thy	Thu Nov 13 17:19:52 2014 +0100
@@ -29,6 +29,9 @@
   unfolding pair_measure_def using pair_measure_closed[of A B]
   by (rule space_measure_of)
 
+lemma SIGMA_Collect_eq: "(SIGMA x:space M. {y\<in>space N. P x y}) = {x\<in>space (M \<Otimes>\<^sub>M N). P (fst x) (snd x)}"
+  by (auto simp: space_pair_measure)
+
 lemma sets_pair_measure:
   "sets (A \<Otimes>\<^sub>M B) = sigma_sets (space A \<times> space B) {a \<times> b | a b. a \<in> sets A \<and> b \<in> sets B}"
   unfolding pair_measure_def using pair_measure_closed[of A B]