src/HOL/Probability/Bochner_Integration.thy
changeset 57447 87429bdecad5
parent 57418 6ab1c7cb0b8d
child 57512 cc97b347b301
equal deleted inserted replaced
57446:06e195515deb 57447:87429bdecad5
  1646     by (cases "\<integral>\<^sup>+ x. ereal (f x) \<partial>M") (auto intro!: integrableI_nn_integral_finite assms)
  1646     by (cases "\<integral>\<^sup>+ x. ereal (f x) \<partial>M") (auto intro!: integrableI_nn_integral_finite assms)
  1647   from nn_integral_eq_integral[OF this nonneg] show ?thesis
  1647   from nn_integral_eq_integral[OF this nonneg] show ?thesis
  1648     by simp
  1648     by simp
  1649 qed
  1649 qed
  1650   
  1650   
       
  1651 lemma has_bochner_integral_nn_integral:
       
  1652   assumes "f \<in> borel_measurable M" "AE x in M. 0 \<le> f x"
       
  1653   assumes "(\<integral>\<^sup>+x. f x \<partial>M) = ereal x"
       
  1654   shows "has_bochner_integral M f x"
       
  1655   unfolding has_bochner_integral_iff
       
  1656   using assms by (auto simp: assms integral_eq_nn_integral intro: integrableI_nn_integral_finite)
       
  1657 
  1651 lemma integrableI_simple_bochner_integrable:
  1658 lemma integrableI_simple_bochner_integrable:
  1652   fixes f :: "'a \<Rightarrow> 'b::{banach, second_countable_topology}"
  1659   fixes f :: "'a \<Rightarrow> 'b::{banach, second_countable_topology}"
  1653   shows "simple_bochner_integrable M f \<Longrightarrow> integrable M f"
  1660   shows "simple_bochner_integrable M f \<Longrightarrow> integrable M f"
  1654   by (intro integrableI_sequence[where s="\<lambda>_. f"] borel_measurable_simple_function)
  1661   by (intro integrableI_sequence[where s="\<lambda>_. f"] borel_measurable_simple_function)
  1655      (auto simp: zero_ereal_def[symmetric] simple_bochner_integrable.simps)
  1662      (auto simp: zero_ereal_def[symmetric] simple_bochner_integrable.simps)