src/HOL/Probability/Bochner_Integration.thy
changeset 63092 a949b2a5f51d
parent 63040 eb4ddd18d635
child 63566 e5abbdee461a
equal deleted inserted replaced
63091:54f16a0a3069 63092:a949b2a5f51d
   941   "integrable M f \<Longrightarrow> g \<in> measurable N M \<Longrightarrow> (\<lambda>x. f (g x)) \<in> borel_measurable N"
   941   "integrable M f \<Longrightarrow> g \<in> measurable N M \<Longrightarrow> (\<lambda>x. f (g x)) \<in> borel_measurable N"
   942   using borel_measurable_integrable[measurable] by measurable
   942   using borel_measurable_integrable[measurable] by measurable
   943 
   943 
   944 lemma integrable_cong:
   944 lemma integrable_cong:
   945   "M = N \<Longrightarrow> (\<And>x. x \<in> space N \<Longrightarrow> f x = g x) \<Longrightarrow> integrable M f \<longleftrightarrow> integrable N g"
   945   "M = N \<Longrightarrow> (\<And>x. x \<in> space N \<Longrightarrow> f x = g x) \<Longrightarrow> integrable M f \<longleftrightarrow> integrable N g"
   946   using assms by (simp cong: has_bochner_integral_cong add: integrable.simps)
   946   by (simp cong: has_bochner_integral_cong add: integrable.simps)
   947 
   947 
   948 lemma integrable_cong_AE:
   948 lemma integrable_cong_AE:
   949   "f \<in> borel_measurable M \<Longrightarrow> g \<in> borel_measurable M \<Longrightarrow> AE x in M. f x = g x \<Longrightarrow>
   949   "f \<in> borel_measurable M \<Longrightarrow> g \<in> borel_measurable M \<Longrightarrow> AE x in M. f x = g x \<Longrightarrow>
   950     integrable M f \<longleftrightarrow> integrable M g"
   950     integrable M f \<longleftrightarrow> integrable M g"
   951   unfolding integrable.simps
   951   unfolding integrable.simps
   952   by (intro has_bochner_integral_cong_AE arg_cong[where f=Ex] ext)
   952   by (intro has_bochner_integral_cong_AE arg_cong[where f=Ex] ext)
   953 
   953 
   954 lemma integral_cong:
   954 lemma integral_cong:
   955   "M = N \<Longrightarrow> (\<And>x. x \<in> space N \<Longrightarrow> f x = g x) \<Longrightarrow> integral\<^sup>L M f = integral\<^sup>L N g"
   955   "M = N \<Longrightarrow> (\<And>x. x \<in> space N \<Longrightarrow> f x = g x) \<Longrightarrow> integral\<^sup>L M f = integral\<^sup>L N g"
   956   using assms by (simp cong: has_bochner_integral_cong cong del: if_cong add: lebesgue_integral_def)
   956   by (simp cong: has_bochner_integral_cong cong del: if_cong add: lebesgue_integral_def)
   957 
   957 
   958 lemma integral_cong_AE:
   958 lemma integral_cong_AE:
   959   "f \<in> borel_measurable M \<Longrightarrow> g \<in> borel_measurable M \<Longrightarrow> AE x in M. f x = g x \<Longrightarrow>
   959   "f \<in> borel_measurable M \<Longrightarrow> g \<in> borel_measurable M \<Longrightarrow> AE x in M. f x = g x \<Longrightarrow>
   960     integral\<^sup>L M f = integral\<^sup>L M g"
   960     integral\<^sup>L M f = integral\<^sup>L M g"
   961   unfolding lebesgue_integral_def
   961   unfolding lebesgue_integral_def