src/HOL/Probability/Caratheodory.thy
changeset 55642 63beb38e9258
parent 52141 eff000cab70f
child 56166 9a241bc276cd
equal deleted inserted replaced
55641:5b466efedd2c 55642:63beb38e9258
   526       fix x i
   526       fix x i
   527       assume x: "x \<in> A i"
   527       assume x: "x \<in> A i"
   528       with sbBB [of i] obtain j where "x \<in> BB i j"
   528       with sbBB [of i] obtain j where "x \<in> BB i j"
   529         by blast
   529         by blast
   530       thus "\<exists>i. x \<in> split BB (prod_decode i)"
   530       thus "\<exists>i. x \<in> split BB (prod_decode i)"
   531         by (metis prod_encode_inverse prod.cases)
   531         by (metis prod_encode_inverse prod.case)
   532     qed
   532     qed
   533     have "(f \<circ> C) = (f \<circ> (\<lambda>(x, y). BB x y)) \<circ> prod_decode"
   533     have "(f \<circ> C) = (f \<circ> (\<lambda>(x, y). BB x y)) \<circ> prod_decode"
   534       by (rule ext)  (auto simp add: C_def)
   534       by (rule ext)  (auto simp add: C_def)
   535     moreover have "suminf ... = (\<Sum>n. \<Sum>i. f (BB n i))" using BBle
   535     moreover have "suminf ... = (\<Sum>n. \<Sum>i. f (BB n i))" using BBle
   536       using BB posf[unfolded positive_def]
   536       using BB posf[unfolded positive_def]