src/HOL/Analysis/Finite_Product_Measure.thy
changeset 69313 b021008c5397
parent 69260 0a9688695a1b
child 69517 dc20f278e8f3
--- a/src/HOL/Analysis/Finite_Product_Measure.thy	Sun Nov 18 09:51:41 2018 +0100
+++ b/src/HOL/Analysis/Finite_Product_Measure.thy	Sun Nov 18 18:07:51 2018 +0000
@@ -779,7 +779,7 @@
   show ?case
   proof (intro exI[of _ "\<Union>i. J i"] bexI[of _ "\<Union>i. prod_emb (\<Union>i. J i) M (J i) (X i)"] conjI)
     show "(\<Union>i. J i) \<subseteq> I" "countable (\<Union>i. J i)" using J by auto
-    with J show "UNION UNIV K = prod_emb I M (\<Union>i. J i) (\<Union>i. prod_emb (\<Union>i. J i) M (J i) (X i))"
+    with J show "\<Union>(K ` UNIV) = prod_emb I M (\<Union>i. J i) (\<Union>i. prod_emb (\<Union>i. J i) M (J i) (X i))"
       by (simp add: K[abs_def] SUP_upper)
   qed(auto intro: X)
 qed