src/HOL/Probability/Radon_Nikodym.thy
changeset 52141 eff000cab70f
parent 51329 4a3c453f99a1
child 53015 a1119cf551e8
--- a/src/HOL/Probability/Radon_Nikodym.thy	Sat May 25 15:44:08 2013 +0200
+++ b/src/HOL/Probability/Radon_Nikodym.thy	Sat May 25 15:44:29 2013 +0200
@@ -571,9 +571,9 @@
     show "(SUP i. emeasure M (?O i)) \<le> ?a" unfolding SUP_def
     proof (safe intro!: Sup_mono, unfold bex_simps)
       fix i
-      have *: "(\<Union>Q' ` {..i}) = ?O i" by auto
+      have *: "(\<Union>(Q' ` {..i})) = ?O i" by auto
       then show "\<exists>x. (x \<in> sets M \<and> N x \<noteq> \<infinity>) \<and>
-        emeasure M (\<Union>Q' ` {..i}) \<le> emeasure M x"
+        emeasure M (\<Union>(Q' ` {..i})) \<le> emeasure M x"
         using O_in_G[of i] by (auto intro!: exI[of _ "?O i"])
     qed
   qed