author | paulson <lp15@cam.ac.uk> |
Tue, 13 Oct 2015 14:49:15 +0100 | |
changeset 61427 | 3c69ea85f8dd |
parent 61426 | d53db136e8fd |
child 61428 | 5e1938107371 |
--- a/src/HOL/Probability/Caratheodory.thy Tue Oct 13 12:42:08 2015 +0100 +++ b/src/HOL/Probability/Caratheodory.thy Tue Oct 13 14:49:15 2015 +0100 @@ -649,7 +649,7 @@ with \<mu>'_spec[THEN bspec, of "\<Union>C"] obtain D where D: "D \<subseteq> M" "finite D" "disjoint D" "\<Union>C = \<Union>D" and "\<mu>' (\<Union>C) = (\<Sum>d\<in>D. \<mu> d)" - by blast + by auto with sum_eq[OF C D] have "\<mu>' (\<Union>C) = (\<Sum>c\<in>C. \<mu> c)" by simp } note \<mu>' = this