src/HOL/Probability/Radon_Nikodym.thy
changeset 45769 2d5b1af2426a
parent 44941 617eb31e63f9
child 45777 c36637603821
equal deleted inserted replaced
45768:97be233b32ed 45769:2d5b1af2426a
  1095       proof (cases "f x")
  1095       proof (cases "f x")
  1096         case PInf with x show ?thesis unfolding A_def by (auto intro: exI[of _ 0])
  1096         case PInf with x show ?thesis unfolding A_def by (auto intro: exI[of _ 0])
  1097       next
  1097       next
  1098         case (real r)
  1098         case (real r)
  1099         with less_PInf_Ex_of_nat[of "f x"] obtain n :: nat where "f x < n" by (auto simp: real_eq_of_nat)
  1099         with less_PInf_Ex_of_nat[of "f x"] obtain n :: nat where "f x < n" by (auto simp: real_eq_of_nat)
  1100         then show ?thesis using x real unfolding A_def by (auto intro!: exI[of _ "Suc n"])
  1100         then show ?thesis using x real unfolding A_def by (auto intro!: exI[of _ "Suc n"] simp: real_eq_of_nat)
  1101       next
  1101       next
  1102         case MInf with x show ?thesis
  1102         case MInf with x show ?thesis
  1103           unfolding A_def by (auto intro!: exI[of _ "Suc 0"])
  1103           unfolding A_def by (auto intro!: exI[of _ "Suc 0"])
  1104       qed
  1104       qed
  1105     qed (auto simp: A_def)
  1105     qed (auto simp: A_def)
  1115       from positive_integral_cong_AE[OF this] show ?thesis by simp
  1115       from positive_integral_cong_AE[OF this] show ?thesis by simp
  1116     next
  1116     next
  1117       case (Suc n)
  1117       case (Suc n)
  1118       then have "(\<integral>\<^isup>+x. f x * indicator (A i \<inter> Q j) x \<partial>M) \<le>
  1118       then have "(\<integral>\<^isup>+x. f x * indicator (A i \<inter> Q j) x \<partial>M) \<le>
  1119         (\<integral>\<^isup>+x. (Suc n :: ereal) * indicator (Q j) x \<partial>M)"
  1119         (\<integral>\<^isup>+x. (Suc n :: ereal) * indicator (Q j) x \<partial>M)"
  1120         by (auto intro!: positive_integral_mono simp: indicator_def A_def)
  1120         by (auto intro!: positive_integral_mono simp: indicator_def A_def real_eq_of_nat)
  1121       also have "\<dots> = Suc n * \<mu> (Q j)"
  1121       also have "\<dots> = Suc n * \<mu> (Q j)"
  1122         using Q by (auto intro!: positive_integral_cmult_indicator)
  1122         using Q by (auto intro!: positive_integral_cmult_indicator)
  1123       also have "\<dots> < \<infinity>"
  1123       also have "\<dots> < \<infinity>"
  1124         using Q by (auto simp: real_eq_of_nat[symmetric])
  1124         using Q by (auto simp: real_eq_of_nat[symmetric])
  1125       finally show ?thesis by simp
  1125       finally show ?thesis by simp