src/HOL/Analysis/Nonnegative_Lebesgue_Integration.thy
changeset 66804 3f9bb52082c4
parent 65680 378a2f11bec9
child 67399 eab6ce8368fa
--- a/src/HOL/Analysis/Nonnegative_Lebesgue_Integration.thy	Sun Oct 08 22:28:20 2017 +0200
+++ b/src/HOL/Analysis/Nonnegative_Lebesgue_Integration.thy	Sun Oct 08 22:28:20 2017 +0200
@@ -648,7 +648,7 @@
       if \<exists>x\<in>space M. y = f x \<and> z = g x then y * emeasure M {x\<in>space M. g x = z} else 0))"
     by (auto intro!: sum.cong simp: sum_distrib_left)
   also have "\<dots> = ?r"
-    by (subst sum.commute)
+    by (subst sum.swap)
        (auto intro!: sum.cong simp: sum.If_cases scaleR_sum_right[symmetric] eq)
   finally show "integral\<^sup>S M f = ?r" .
 qed