src/HOL/Probability/Finite_Product_Measure.thy
changeset 57512 cc97b347b301
parent 57447 87429bdecad5
child 58606 9c66f7c541fb
--- a/src/HOL/Probability/Finite_Product_Measure.thy	Fri Jul 04 20:07:08 2014 +0200
+++ b/src/HOL/Probability/Finite_Product_Measure.thy	Fri Jul 04 20:18:47 2014 +0200
@@ -643,7 +643,7 @@
       using E by (subst insert) (auto intro!: setprod.cong)
     also have "(\<Prod>j\<in>I. if j \<in> J - {i} then emeasure (M j) (E j) else emeasure (M j) (space (M j))) *
        emeasure (M i) (if i \<in> J then E i else space (M i)) = (\<Prod>j\<in>insert i I. ?f J E j)"
-      using insert by (auto simp: mult_commute intro!: arg_cong2[where f="op *"] setprod.cong)
+      using insert by (auto simp: mult.commute intro!: arg_cong2[where f="op *"] setprod.cong)
     also have "\<dots> = (\<Prod>j\<in>J \<union> ?I. ?f J E j)"
       using insert(1,2) J E by (intro setprod.mono_neutral_right) auto
     finally show "?\<mu> ?p = \<dots>" .