src/HOL/Probability/Sigma_Algebra.thy
changeset 60063 81835db730e8
parent 59415 854fe701c984
child 60727 53697011b03a
equal deleted inserted replaced
60062:4c5de5a860ee 60063:81835db730e8
  2359     by (intro image_cong) (auto dest: sets.sets_into_space)
  2359     by (intro image_cong) (auto dest: sets.sets_into_space)
  2360   ultimately show "sigma_sets (\<Omega> \<inter> space M) (op \<inter> \<Omega> ` sets M) = op \<inter> \<Omega> ` sets M"
  2360   ultimately show "sigma_sets (\<Omega> \<inter> space M) (op \<inter> \<Omega> ` sets M) = op \<inter> \<Omega> ` sets M"
  2361     by simp
  2361     by simp
  2362 qed
  2362 qed
  2363 
  2363 
       
  2364 lemma sets_restrict_space_count_space :
       
  2365   "sets (restrict_space (count_space A) B) = sets (count_space (A \<inter> B))"
       
  2366 by(auto simp add: sets_restrict_space)
       
  2367 
  2364 lemma sets_restrict_UNIV[simp]: "sets (restrict_space M UNIV) = sets M"
  2368 lemma sets_restrict_UNIV[simp]: "sets (restrict_space M UNIV) = sets M"
  2365   by (auto simp add: sets_restrict_space)
  2369   by (auto simp add: sets_restrict_space)
  2366 
  2370 
  2367 lemma sets_restrict_restrict_space:
  2371 lemma sets_restrict_restrict_space:
  2368   "sets (restrict_space (restrict_space M A) B) = sets (restrict_space M (A \<inter> B))"
  2372   "sets (restrict_space (restrict_space M A) B) = sets (restrict_space M (A \<inter> B))"