src/HOL/Analysis/Bochner_Integration.thy
changeset 69144 f13b82281715
parent 69064 5840724b1d71
child 69546 27dae626822b
equal deleted inserted replaced
69143:5acb1eece41b 69144:f13b82281715
  2850   have [simp]: "\<And>x. x \<in> space N \<Longrightarrow> integrable M (f x) \<longleftrightarrow> (\<integral>\<^sup>+y. norm (f x y) \<partial>M) < \<infinity>"
  2850   have [simp]: "\<And>x. x \<in> space N \<Longrightarrow> integrable M (f x) \<longleftrightarrow> (\<integral>\<^sup>+y. norm (f x y) \<partial>M) < \<infinity>"
  2851     unfolding integrable_iff_bounded by simp
  2851     unfolding integrable_iff_bounded by simp
  2852   show ?thesis
  2852   show ?thesis
  2853     by (simp cong: measurable_cong)
  2853     by (simp cong: measurable_cong)
  2854 qed
  2854 qed
  2855 
       
  2856 lemma%unimportant Collect_subset [simp]: "{x\<in>A. P x} \<subseteq> A" by auto
       
  2857 
  2855 
  2858 lemma%unimportant (in sigma_finite_measure) measurable_measure[measurable (raw)]:
  2856 lemma%unimportant (in sigma_finite_measure) measurable_measure[measurable (raw)]:
  2859   "(\<And>x. x \<in> space N \<Longrightarrow> A x \<subseteq> space M) \<Longrightarrow>
  2857   "(\<And>x. x \<in> space N \<Longrightarrow> A x \<subseteq> space M) \<Longrightarrow>
  2860     {x \<in> space (N \<Otimes>\<^sub>M M). snd x \<in> A (fst x)} \<in> sets (N \<Otimes>\<^sub>M M) \<Longrightarrow>
  2858     {x \<in> space (N \<Otimes>\<^sub>M M). snd x \<in> A (fst x)} \<in> sets (N \<Otimes>\<^sub>M M) \<Longrightarrow>
  2861     (\<lambda>x. measure M (A x)) \<in> borel_measurable N"
  2859     (\<lambda>x. measure M (A x)) \<in> borel_measurable N"