src/HOL/Analysis/Borel_Space.thy
changeset 64911 f0e07600de47
parent 64320 ba194424b895
child 66164 2d79288b042c
equal deleted inserted replaced
64910:6108dddad9f0 64911:f0e07600de47
  2124   fixes p::real
  2124   fixes p::real
  2125   assumes [measurable]: "f \<in> borel_measurable M"
  2125   assumes [measurable]: "f \<in> borel_measurable M"
  2126   shows "(\<lambda>x. \<bar>f x\<bar> powr p) \<in> borel_measurable M"
  2126   shows "(\<lambda>x. \<bar>f x\<bar> powr p) \<in> borel_measurable M"
  2127 unfolding powr_def by auto
  2127 unfolding powr_def by auto
  2128 
  2128 
  2129 text {* The next one is a variation around \verb+measurable_restrict_space+.*}
  2129 text \<open>The next one is a variation around \verb+measurable_restrict_space+.\<close>
  2130 
  2130 
  2131 lemma measurable_restrict_space3:
  2131 lemma measurable_restrict_space3:
  2132   assumes "f \<in> measurable M N" and
  2132   assumes "f \<in> measurable M N" and
  2133           "f \<in> A \<rightarrow> B"
  2133           "f \<in> A \<rightarrow> B"
  2134   shows "f \<in> measurable (restrict_space M A) (restrict_space N B)"
  2134   shows "f \<in> measurable (restrict_space M A) (restrict_space N B)"
  2136   have "f \<in> measurable (restrict_space M A) N" using assms(1) measurable_restrict_space1 by auto
  2136   have "f \<in> measurable (restrict_space M A) N" using assms(1) measurable_restrict_space1 by auto
  2137   then show ?thesis by (metis Int_iff funcsetI funcset_mem
  2137   then show ?thesis by (metis Int_iff funcsetI funcset_mem
  2138       measurable_restrict_space2[of f, of "restrict_space M A", of B, of N] assms(2) space_restrict_space)
  2138       measurable_restrict_space2[of f, of "restrict_space M A", of B, of N] assms(2) space_restrict_space)
  2139 qed
  2139 qed
  2140 
  2140 
  2141 text {* The next one is a variation around \verb+measurable_piecewise_restrict+.*}
  2141 text \<open>The next one is a variation around \verb+measurable_piecewise_restrict+.\<close>
  2142 
  2142 
  2143 lemma measurable_piecewise_restrict2:
  2143 lemma measurable_piecewise_restrict2:
  2144   assumes [measurable]: "\<And>n. A n \<in> sets M"
  2144   assumes [measurable]: "\<And>n. A n \<in> sets M"
  2145       and "space M = (\<Union>(n::nat). A n)"
  2145       and "space M = (\<Union>(n::nat). A n)"
  2146           "\<And>n. \<exists>h \<in> measurable M N. (\<forall>x \<in> A n. f x = h x)"
  2146           "\<And>n. \<exists>h \<in> measurable M N. (\<forall>x \<in> A n. f x = h x)"
  2160   ultimately show "f-`B \<inter> space M \<in> sets M" by simp
  2160   ultimately show "f-`B \<inter> space M \<in> sets M" by simp
  2161 next
  2161 next
  2162   fix x assume "x \<in> space M"
  2162   fix x assume "x \<in> space M"
  2163   then obtain n where "x \<in> A n" using assms(2) by blast
  2163   then obtain n where "x \<in> A n" using assms(2) by blast
  2164   obtain h where [measurable]: "h \<in> measurable M N" and "\<forall>x \<in> A n. f x = h x" using assms(3) by blast
  2164   obtain h where [measurable]: "h \<in> measurable M N" and "\<forall>x \<in> A n. f x = h x" using assms(3) by blast
  2165   then have "f x = h x" using `x \<in> A n` by blast
  2165   then have "f x = h x" using \<open>x \<in> A n\<close> by blast
  2166   moreover have "h x \<in> space N" by (metis measurable_space `x \<in> space M` `h \<in> measurable M N`)
  2166   moreover have "h x \<in> space N" by (metis measurable_space \<open>x \<in> space M\<close> \<open>h \<in> measurable M N\<close>)
  2167   ultimately show "f x \<in> space N" by simp
  2167   ultimately show "f x \<in> space N" by simp
  2168 qed
  2168 qed
  2169 
  2169 
  2170 end
  2170 end