src/HOL/Probability/Bochner_Integration.thy
changeset 57447 87429bdecad5
parent 57418 6ab1c7cb0b8d
child 57512 cc97b347b301
--- a/src/HOL/Probability/Bochner_Integration.thy	Mon Jun 30 15:45:03 2014 +0200
+++ b/src/HOL/Probability/Bochner_Integration.thy	Mon Jun 30 15:45:21 2014 +0200
@@ -1648,6 +1648,13 @@
     by simp
 qed
   
+lemma has_bochner_integral_nn_integral:
+  assumes "f \<in> borel_measurable M" "AE x in M. 0 \<le> f x"
+  assumes "(\<integral>\<^sup>+x. f x \<partial>M) = ereal x"
+  shows "has_bochner_integral M f x"
+  unfolding has_bochner_integral_iff
+  using assms by (auto simp: assms integral_eq_nn_integral intro: integrableI_nn_integral_finite)
+
 lemma integrableI_simple_bochner_integrable:
   fixes f :: "'a \<Rightarrow> 'b::{banach, second_countable_topology}"
   shows "simple_bochner_integrable M f \<Longrightarrow> integrable M f"