src/HOL/Probability/Lebesgue_Integration.thy
changeset 56213 e5720d3c18f0
parent 56212 3253aaf73a01
child 56218 1c3f1f2431f9
--- a/src/HOL/Probability/Lebesgue_Integration.thy	Tue Mar 18 22:11:46 2014 +0100
+++ b/src/HOL/Probability/Lebesgue_Integration.thy	Wed Mar 19 15:34:57 2014 +0100
@@ -2239,7 +2239,7 @@
   proof eventually_elim
     fix j x assume [simp]: "x \<in> space M"
     have "\<bar>\<Sum>i<j. f i x\<bar> \<le> (\<Sum>i<j. \<bar>f i x\<bar>)" by (rule setsum_abs)
-    also have "\<dots> \<le> w x" using w[of x] series_pos_le[of "\<lambda>i. \<bar>f i x\<bar>"] unfolding sums_iff by auto
+    also have "\<dots> \<le> w x" using w[of x] setsum_le_suminf[of "\<lambda>i. \<bar>f i x\<bar>"] unfolding sums_iff by auto
     finally show "\<bar>\<Sum>i<j. f i x\<bar> \<le> ?w x" by simp
   qed