src/HOL/Analysis/Radon_Nikodym.thy
changeset 69745 aec42cee2521
parent 69739 8b47c021666e
child 70136 f03a01a18c6e
equal deleted inserted replaced
69744:bb0a354f6b46 69745:aec42cee2521
   835     show "countable (range (\<lambda>(i, j). A i \<inter> Q j))"
   835     show "countable (range (\<lambda>(i, j). A i \<inter> Q j))"
   836       by auto
   836       by auto
   837     show "range (\<lambda>(i, j). A i \<inter> Q j) \<subseteq> sets (density M f)"
   837     show "range (\<lambda>(i, j). A i \<inter> Q j) \<subseteq> sets (density M f)"
   838       using A_in_sets by auto
   838       using A_in_sets by auto
   839   next
   839   next
   840     have "\<Union>range (\<lambda>(i, j). A i \<inter> Q j) = (\<Union>i j. A i \<inter> Q j)"
   840     have "\<Union>(range (\<lambda>(i, j). A i \<inter> Q j)) = (\<Union>i j. A i \<inter> Q j)"
   841       by auto
   841       by auto
   842     also have "\<dots> = (\<Union>i. A i) \<inter> space M" using Q by auto
   842     also have "\<dots> = (\<Union>i. A i) \<inter> space M" using Q by auto
   843     also have "(\<Union>i. A i) = space M"
   843     also have "(\<Union>i. A i) = space M"
   844     proof safe
   844     proof safe
   845       fix x assume x: "x \<in> space M"
   845       fix x assume x: "x \<in> space M"
   854           by simp
   854           by simp
   855         finally show ?thesis
   855         finally show ?thesis
   856           using x real by (auto simp: A_def ennreal_of_nat_eq_real_of_nat intro!: exI[of _ "Suc n"])
   856           using x real by (auto simp: A_def ennreal_of_nat_eq_real_of_nat intro!: exI[of _ "Suc n"])
   857       qed
   857       qed
   858     qed (auto simp: A_def)
   858     qed (auto simp: A_def)
   859     finally show "\<Union>range (\<lambda>(i, j). A i \<inter> Q j) = space ?N" by simp
   859     finally show "\<Union>(range (\<lambda>(i, j). A i \<inter> Q j)) = space ?N" by simp
   860   next
   860   next
   861     fix X assume "X \<in> range (\<lambda>(i, j). A i \<inter> Q j)"
   861     fix X assume "X \<in> range (\<lambda>(i, j). A i \<inter> Q j)"
   862     then obtain i j where [simp]:"X = A i \<inter> Q j" by auto
   862     then obtain i j where [simp]:"X = A i \<inter> Q j" by auto
   863     have "(\<integral>\<^sup>+x. f x * indicator (A i \<inter> Q j) x \<partial>M) \<noteq> \<infinity>"
   863     have "(\<integral>\<^sup>+x. f x * indicator (A i \<inter> Q j) x \<partial>M) \<noteq> \<infinity>"
   864     proof (cases i)
   864     proof (cases i)