src/HOL/Analysis/Borel_Space.thy
changeset 64267 b9a1486e79be
parent 64008 17a20ca86d62
child 64272 f76b6dda2e56
equal deleted inserted replaced
64265:8eb6365f5916 64267:b9a1486e79be
   967   assumes f: "f \<in> borel_measurable M"
   967   assumes f: "f \<in> borel_measurable M"
   968   assumes g: "g \<in> borel_measurable M"
   968   assumes g: "g \<in> borel_measurable M"
   969   shows "(\<lambda>x. f x + g x) \<in> borel_measurable M"
   969   shows "(\<lambda>x. f x + g x) \<in> borel_measurable M"
   970   using f g by (rule borel_measurable_continuous_Pair) (intro continuous_intros)
   970   using f g by (rule borel_measurable_continuous_Pair) (intro continuous_intros)
   971 
   971 
   972 lemma borel_measurable_setsum[measurable (raw)]:
   972 lemma borel_measurable_sum[measurable (raw)]:
   973   fixes f :: "'c \<Rightarrow> 'a \<Rightarrow> 'b::{second_countable_topology, topological_comm_monoid_add}"
   973   fixes f :: "'c \<Rightarrow> 'a \<Rightarrow> 'b::{second_countable_topology, topological_comm_monoid_add}"
   974   assumes "\<And>i. i \<in> S \<Longrightarrow> f i \<in> borel_measurable M"
   974   assumes "\<And>i. i \<in> S \<Longrightarrow> f i \<in> borel_measurable M"
   975   shows "(\<lambda>x. \<Sum>i\<in>S. f i x) \<in> borel_measurable M"
   975   shows "(\<lambda>x. \<Sum>i\<in>S. f i x) \<in> borel_measurable M"
   976 proof cases
   976 proof cases
   977   assume "finite S"
   977   assume "finite S"
  1644   assumes "g \<in> borel_measurable M"
  1644   assumes "g \<in> borel_measurable M"
  1645   shows borel_measurable_ereal_diff: "(\<lambda>x. f x - g x) \<in> borel_measurable M"
  1645   shows borel_measurable_ereal_diff: "(\<lambda>x. f x - g x) \<in> borel_measurable M"
  1646     and borel_measurable_ereal_divide: "(\<lambda>x. f x / g x) \<in> borel_measurable M"
  1646     and borel_measurable_ereal_divide: "(\<lambda>x. f x / g x) \<in> borel_measurable M"
  1647   using assms by (simp_all add: minus_ereal_def divide_ereal_def)
  1647   using assms by (simp_all add: minus_ereal_def divide_ereal_def)
  1648 
  1648 
  1649 lemma borel_measurable_ereal_setsum[measurable (raw)]:
  1649 lemma borel_measurable_ereal_sum[measurable (raw)]:
  1650   fixes f :: "'c \<Rightarrow> 'a \<Rightarrow> ereal"
  1650   fixes f :: "'c \<Rightarrow> 'a \<Rightarrow> ereal"
  1651   assumes "\<And>i. i \<in> S \<Longrightarrow> f i \<in> borel_measurable M"
  1651   assumes "\<And>i. i \<in> S \<Longrightarrow> f i \<in> borel_measurable M"
  1652   shows "(\<lambda>x. \<Sum>i\<in>S. f i x) \<in> borel_measurable M"
  1652   shows "(\<lambda>x. \<Sum>i\<in>S. f i x) \<in> borel_measurable M"
  1653   using assms by (induction S rule: infinite_finite_induct) auto
  1653   using assms by (induction S rule: infinite_finite_induct) auto
  1654 
  1654