add measurable_compose
authorhoelzl
Wed, 10 Oct 2012 12:12:22 +0200
changeset 49782 d5c6a905b57e
parent 49781 59b219ca3513
child 49783 38b84d1802ed
add measurable_compose
src/HOL/Probability/Sigma_Algebra.thy
--- a/src/HOL/Probability/Sigma_Algebra.thy	Wed Oct 10 12:12:21 2012 +0200
+++ b/src/HOL/Probability/Sigma_Algebra.thy	Wed Oct 10 12:12:22 2012 +0200
@@ -1310,6 +1310,10 @@
   apply force+
   done
 
+lemma measurable_compose:
+  "f \<in> measurable M N \<Longrightarrow> g \<in> measurable N L \<Longrightarrow> (\<lambda>x. g (f x)) \<in> measurable M L"
+  using measurable_comp[of f M N g L] by (simp add: comp_def)
+
 lemma measurable_Least:
   assumes meas: "\<And>i::nat. {x\<in>space M. P i x} \<in> M"
   shows "(\<lambda>x. LEAST j. P j x) -` A \<inter> space M \<in> sets M"