src/HOL/Analysis/Sigma_Algebra.thy
changeset 64008 17a20ca86d62
parent 63627 6ddb43c6b711
child 66453 cc19f7ca2ed6
equal deleted inserted replaced
64007:041cda506fb2 64008:17a20ca86d62
  1242 definition "Int_stable M \<longleftrightarrow> (\<forall> a \<in> M. \<forall> b \<in> M. a \<inter> b \<in> M)"
  1242 definition "Int_stable M \<longleftrightarrow> (\<forall> a \<in> M. \<forall> b \<in> M. a \<inter> b \<in> M)"
  1243 
  1243 
  1244 lemma (in algebra) Int_stable: "Int_stable M"
  1244 lemma (in algebra) Int_stable: "Int_stable M"
  1245   unfolding Int_stable_def by auto
  1245   unfolding Int_stable_def by auto
  1246 
  1246 
       
  1247 lemma Int_stableI_image:
       
  1248   "(\<And>i j. i \<in> I \<Longrightarrow> j \<in> I \<Longrightarrow> \<exists>k\<in>I. A i \<inter> A j = A k) \<Longrightarrow> Int_stable (A ` I)"
       
  1249   by (auto simp: Int_stable_def image_def)
       
  1250 
  1247 lemma Int_stableI:
  1251 lemma Int_stableI:
  1248   "(\<And>a b. a \<in> A \<Longrightarrow> b \<in> A \<Longrightarrow> a \<inter> b \<in> A) \<Longrightarrow> Int_stable A"
  1252   "(\<And>a b. a \<in> A \<Longrightarrow> b \<in> A \<Longrightarrow> a \<inter> b \<in> A) \<Longrightarrow> Int_stable A"
  1249   unfolding Int_stable_def by auto
  1253   unfolding Int_stable_def by auto
  1250 
  1254 
  1251 lemma Int_stableD:
  1255 lemma Int_stableD:
  1572   shows sets_measure_of: "sets (measure_of \<Omega> A \<mu>) = sigma_sets \<Omega> A"
  1576   shows sets_measure_of: "sets (measure_of \<Omega> A \<mu>) = sigma_sets \<Omega> A"
  1573     and space_measure_of: "space (measure_of \<Omega> A \<mu>) = \<Omega>"
  1577     and space_measure_of: "space (measure_of \<Omega> A \<mu>) = \<Omega>"
  1574 using assms
  1578 using assms
  1575 by(simp_all add: sets_measure_of_conv space_measure_of_conv)
  1579 by(simp_all add: sets_measure_of_conv space_measure_of_conv)
  1576 
  1580 
       
  1581 lemma space_in_measure_of[simp]: "\<Omega> \<in> sets (measure_of \<Omega> M \<mu>)"
       
  1582   by (subst sets_measure_of_conv) (auto simp: sigma_sets_top)
       
  1583 
  1577 lemma (in sigma_algebra) sets_measure_of_eq[simp]: "sets (measure_of \<Omega> M \<mu>) = M"
  1584 lemma (in sigma_algebra) sets_measure_of_eq[simp]: "sets (measure_of \<Omega> M \<mu>) = M"
  1578   using space_closed by (auto intro!: sigma_sets_eq)
  1585   using space_closed by (auto intro!: sigma_sets_eq)
  1579 
  1586 
  1580 lemma (in sigma_algebra) space_measure_of_eq[simp]: "space (measure_of \<Omega> M \<mu>) = \<Omega>"
  1587 lemma (in sigma_algebra) space_measure_of_eq[simp]: "space (measure_of \<Omega> M \<mu>) = \<Omega>"
  1581   by (rule space_measure_of_conv)
  1588   by (rule space_measure_of_conv)
  2257   assumes eq: "\<And>x. x \<in> space M \<Longrightarrow> x \<notin> X \<Longrightarrow> f x = g x"
  2264   assumes eq: "\<And>x. x \<in> space M \<Longrightarrow> x \<notin> X \<Longrightarrow> f x = g x"
  2258   shows "g \<in> measurable M N"
  2265   shows "g \<in> measurable M N"
  2259   by (rule measurable_restrict_countable[OF X])
  2266   by (rule measurable_restrict_countable[OF X])
  2260      (auto simp: eq[symmetric] space_restrict_space cong: measurable_cong' intro: f measurable_restrict_space1)
  2267      (auto simp: eq[symmetric] space_restrict_space cong: measurable_cong' intro: f measurable_restrict_space1)
  2261 
  2268 
       
  2269 lemma measurable_count_space_extend: "A \<subseteq> B \<Longrightarrow> f \<in> space M \<rightarrow> A \<Longrightarrow> f \<in> M \<rightarrow>\<^sub>M count_space B \<Longrightarrow> f \<in> M \<rightarrow>\<^sub>M count_space A"
       
  2270   by (auto simp: measurable_def)
       
  2271 
  2262 end
  2272 end