diff -r e13e70f32407 -r e01015e49041 src/HOL/Probability/Infinite_Product_Measure.thy --- a/src/HOL/Probability/Infinite_Product_Measure.thy Tue Dec 29 22:41:22 2015 +0100 +++ b/src/HOL/Probability/Infinite_Product_Measure.thy Tue Dec 29 23:04:53 2015 +0100 @@ -187,7 +187,7 @@ lemma measure_PiM_countable: fixes E :: "nat \ 'a set" assumes E: "\i. E i \ sets M" - shows "(\n. \i\n. measure M (E i)) ----> measure S (Pi UNIV E)" + shows "(\n. \i\n. measure M (E i)) \ measure S (Pi UNIV E)" proof - let ?E = "\n. emb UNIV {..n} (Pi\<^sub>E {.. n} E)" have "\n. (\i\n. measure M (E i)) = measure S (?E n)"