src/HOL/Probability/Bochner_Integration.thy
changeset 59353 f0707dc3d9aa
parent 59048 7dc8ac6f0895
child 59357 f366643536cd
--- a/src/HOL/Probability/Bochner_Integration.thy	Sun Jan 11 21:06:47 2015 +0100
+++ b/src/HOL/Probability/Bochner_Integration.thy	Tue Jan 13 19:10:36 2015 +0100
@@ -534,9 +534,13 @@
             nn_integral_cong_AE)
      auto
 
-lemma borel_measurable_has_bochner_integral[measurable_dest]:
+lemma borel_measurable_has_bochner_integral:
   "has_bochner_integral M f x \<Longrightarrow> f \<in> borel_measurable M"
-  by (auto elim: has_bochner_integral.cases)
+  by (rule has_bochner_integral.cases)
+
+lemma borel_measurable_has_bochner_integral'[measurable_dest]:
+  "has_bochner_integral M f x \<Longrightarrow> g \<in> measurable N M \<Longrightarrow> (\<lambda>x. f (g x)) \<in> borel_measurable N"
+  using borel_measurable_has_bochner_integral[measurable] by measurable
 
 lemma has_bochner_integral_simple_bochner_integrable:
   "simple_bochner_integrable M f \<Longrightarrow> has_bochner_integral M f (simple_bochner_integral M f)"
@@ -922,6 +926,10 @@
 lemma borel_measurable_integrable[measurable_dest]: "integrable M f \<Longrightarrow> f \<in> borel_measurable M"
   by (auto elim: integrable.cases has_bochner_integral.cases)
 
+lemma borel_measurable_integrable'[measurable_dest]:
+  "integrable M f \<Longrightarrow> g \<in> measurable N M \<Longrightarrow> (\<lambda>x. f (g x)) \<in> borel_measurable N"
+  using borel_measurable_integrable[measurable] by measurable
+
 lemma integrable_cong:
   "M = N \<Longrightarrow> (\<And>x. x \<in> space N \<Longrightarrow> f x = g x) \<Longrightarrow> integrable M f \<longleftrightarrow> integrable N g"
   using assms by (simp cong: has_bochner_integral_cong add: integrable.simps)
@@ -2765,6 +2773,7 @@
   shows "integrable (Pi\<^sub>M I M) (\<lambda>x. (\<Prod>i\<in>I. f i (x i)))" (is "integrable _ ?f")
 proof (unfold integrable_iff_bounded, intro conjI)
   interpret finite_product_sigma_finite M I by default fact
+
   show "?f \<in> borel_measurable (Pi\<^sub>M I M)"
     using assms by simp
   have "(\<integral>\<^sup>+ x. ereal (norm (\<Prod>i\<in>I. f i (x i))) \<partial>Pi\<^sub>M I M) = 
@@ -2854,3 +2863,4 @@
 hide_const simple_bochner_integrable
 
 end
+