src/HOL/Analysis/Finite_Product_Measure.thy
changeset 69745 aec42cee2521
parent 69739 8b47c021666e
child 69918 eddcc7c726f3
--- a/src/HOL/Analysis/Finite_Product_Measure.thy	Sun Jan 27 17:30:09 2019 +0100
+++ b/src/HOL/Analysis/Finite_Product_Measure.thy	Mon Jan 28 10:27:47 2019 +0100
@@ -970,7 +970,7 @@
 
   obtain F where F: "\<And>j. countable (F j)" "\<And>j f. f \<in> F j \<Longrightarrow> f \<in> sets (M j)"
     "\<And>j f. f \<in> F j \<Longrightarrow> emeasure (M j) f \<noteq> \<infinity>" and
-    in_space: "\<And>j. space (M j) = (\<Union>F j)"
+    in_space: "\<And>j. space (M j) = \<Union>(F j)"
     using sigma_finite_countable by (metis subset_eq)
   moreover have "(\<Union>(Pi\<^sub>E I ` Pi\<^sub>E I F)) = space (Pi\<^sub>M I M)"
     using in_space by (auto simp: space_PiM PiE_iff intro!: PiE_choice[THEN iffD2])