src/HOL/Probability/Binary_Product_Measure.thy
changeset 46898 1570b30ee040
parent 46731 5302e932d1e5
child 47694 05663f75964c
--- a/src/HOL/Probability/Binary_Product_Measure.thy	Tue Mar 13 12:51:52 2012 +0100
+++ b/src/HOL/Probability/Binary_Product_Measure.thy	Tue Mar 13 13:31:26 2012 +0100
@@ -197,7 +197,7 @@
 next
   fix A assume "A \<in> sets (M2 \<Otimes>\<^isub>M M1)"
   interpret Q: pair_sigma_algebra M2 M1 by default
-  with Q.sets_pair_sigma_algebra_swap[OF `A \<in> sets (M2 \<Otimes>\<^isub>M M1)`]
+  from Q.sets_pair_sigma_algebra_swap[OF `A \<in> sets (M2 \<Otimes>\<^isub>M M1)`]
   show "?f -` A \<inter> space ?P \<in> sets ?P" by simp
 qed
 
@@ -221,7 +221,7 @@
   assumes Q: "Q \<in> sets P" shows "(\<lambda>x. (x, y)) -` Q \<in> sets M1" (is "?cut Q \<in> sets M1")
 proof -
   interpret Q: pair_sigma_algebra M2 M1 by default
-  with Q.measurable_cut_fst[OF sets_pair_sigma_algebra_swap[OF Q], of y]
+  from Q.measurable_cut_fst[OF sets_pair_sigma_algebra_swap[OF Q], of y]
   show ?thesis by (simp add: vimage_compose[symmetric] comp_def)
 qed