src/HOL/Probability/Sigma_Algebra.thy
changeset 49782 d5c6a905b57e
parent 49773 16907431e477
child 49789 e0a4cb91a8a9
equal deleted inserted replaced
49781:59b219ca3513 49782:d5c6a905b57e
  1308   apply (auto simp add: measurable_def vimage_compose)
  1308   apply (auto simp add: measurable_def vimage_compose)
  1309   apply (subgoal_tac "f -` g -` y \<inter> space a = f -` (g -` y \<inter> space b) \<inter> space a")
  1309   apply (subgoal_tac "f -` g -` y \<inter> space a = f -` (g -` y \<inter> space b) \<inter> space a")
  1310   apply force+
  1310   apply force+
  1311   done
  1311   done
  1312 
  1312 
       
  1313 lemma measurable_compose:
       
  1314   "f \<in> measurable M N \<Longrightarrow> g \<in> measurable N L \<Longrightarrow> (\<lambda>x. g (f x)) \<in> measurable M L"
       
  1315   using measurable_comp[of f M N g L] by (simp add: comp_def)
       
  1316 
  1313 lemma measurable_Least:
  1317 lemma measurable_Least:
  1314   assumes meas: "\<And>i::nat. {x\<in>space M. P i x} \<in> M"
  1318   assumes meas: "\<And>i::nat. {x\<in>space M. P i x} \<in> M"
  1315   shows "(\<lambda>x. LEAST j. P j x) -` A \<inter> space M \<in> sets M"
  1319   shows "(\<lambda>x. LEAST j. P j x) -` A \<inter> space M \<in> sets M"
  1316 proof -
  1320 proof -
  1317   { fix i have "(\<lambda>x. LEAST j. P j x) -` {i} \<inter> space M \<in> sets M"
  1321   { fix i have "(\<lambda>x. LEAST j. P j x) -` {i} \<inter> space M \<in> sets M"