src/HOL/Probability/Sigma_Algebra.thy
changeset 57137 f174712d0a84
parent 57025 e7fd64f82876
child 57138 7b3146180291
--- a/src/HOL/Probability/Sigma_Algebra.thy	Fri May 30 18:13:40 2014 +0200
+++ b/src/HOL/Probability/Sigma_Algebra.thy	Fri May 30 15:56:30 2014 +0200
@@ -2351,9 +2351,9 @@
 qed
 
 lemma measurable_restrict_space2:
-  "\<Omega> \<in> sets N \<Longrightarrow> f \<in> space M \<rightarrow> \<Omega> \<Longrightarrow> f \<in> measurable M N \<Longrightarrow>
+  "\<Omega> \<inter> space N \<in> sets N \<Longrightarrow> f \<in> space M \<rightarrow> \<Omega> \<Longrightarrow> f \<in> measurable M N \<Longrightarrow>
     f \<in> measurable M (restrict_space N \<Omega>)"
-  by (simp add: measurable_def space_restrict_space sets_restrict_space_iff)
+  by (simp add: measurable_def space_restrict_space sets_restrict_space_iff Pi_Int[symmetric])
 
 end