src/HOL/Probability/Infinite_Product_Measure.thy
changeset 51351 dd1dd470690b
parent 50252 4aa34bd43228
child 53015 a1119cf551e8
equal deleted inserted replaced
51350:490f34774a9a 51351:dd1dd470690b
   301         then have "w' \<in> A n" unfolding A_eq using w' by (auto simp: prod_emb_def space_PiM) }
   301         then have "w' \<in> A n" unfolding A_eq using w' by (auto simp: prod_emb_def space_PiM) }
   302       then have "w' \<in> (\<Inter>i. A i)" by auto
   302       then have "w' \<in> (\<Inter>i. A i)" by auto
   303       with `(\<Inter>i. A i) = {}` show False by auto
   303       with `(\<Inter>i. A i) = {}` show False by auto
   304     qed
   304     qed
   305     ultimately show "(\<lambda>i. \<mu>G (A i)) ----> 0"
   305     ultimately show "(\<lambda>i. \<mu>G (A i)) ----> 0"
   306       using LIMSEQ_ereal_INFI[of "\<lambda>i. \<mu>G (A i)"] by simp
   306       using LIMSEQ_INF[of "\<lambda>i. \<mu>G (A i)"] by simp
   307   qed fact+
   307   qed fact+
   308   then guess \<mu> .. note \<mu> = this
   308   then guess \<mu> .. note \<mu> = this
   309   show ?thesis
   309   show ?thesis
   310   proof (subst emeasure_extend_measure_Pair[OF PiM_def, of I M \<mu> J X])
   310   proof (subst emeasure_extend_measure_Pair[OF PiM_def, of I M \<mu> J X])
   311     from assms show "(J \<noteq> {} \<or> I = {}) \<and> finite J \<and> J \<subseteq> I \<and> X \<in> (\<Pi> j\<in>J. sets (M j))"
   311     from assms show "(J \<noteq> {} \<or> I = {}) \<and> finite J \<and> J \<subseteq> I \<and> X \<in> (\<Pi> j\<in>J. sets (M j))"