src/HOL/Probability/Tree_Space.thy
changeset 69313 b021008c5397
parent 69219 d4cec24a1d87
child 69655 2b56cbb02e8a
equal deleted inserted replaced
69312:e0f68a507683 69313:b021008c5397
   195     also have "\<dots> \<in> sets (tree_sigma M)"
   195     also have "\<dots> \<in> sets (tree_sigma M)"
   196       by (intro sets.Diff Compl) auto
   196       by (intro sets.Diff Compl) auto
   197     finally show ?case .
   197     finally show ?case .
   198   next
   198   next
   199     case (Union I)
   199     case (Union I)
   200     have *: "{Node l v r |l v r. (v, l, r) \<in> UNION UNIV I} =
   200     have *: "{Node l v r |l v r. (v, l, r) \<in> \<Union>(I ` UNIV)} =
   201       (\<Union>i. {Node l v r |l v r. (v, l, r) \<in> I i})" by auto
   201       (\<Union>i. {Node l v r |l v r. (v, l, r) \<in> I i})" by auto
   202     show ?case unfolding * using Union(2) by (intro sets.countable_UN) auto
   202     show ?case unfolding * using Union(2) by (intro sets.countable_UN) auto
   203   qed
   203   qed
   204 qed
   204 qed
   205 
   205