src/HOL/Product_Type.thy
changeset 69275 9bbd5497befd
parent 69144 f13b82281715
child 69593 3dda49e08b9d
--- a/src/HOL/Product_Type.thy	Sat Nov 10 07:57:18 2018 +0000
+++ b/src/HOL/Product_Type.thy	Sat Nov 10 07:57:19 2018 +0000
@@ -1049,7 +1049,7 @@
     \<Longrightarrow> A \<subseteq> Collect (case_prod P) \<Longrightarrow> A \<subseteq> Collect (case_prod Q)"
   by fastforce
 
-lemma UN_Times_distrib: "(\<Union>(a, b)\<in>A \<times> B. E a \<times> F b) = UNION A E \<times> UNION B F"
+lemma UN_Times_distrib: "(\<Union>(a, b)\<in>A \<times> B. E a \<times> F b) = \<Union>(E ` A) \<times> \<Union>(F ` B)"
   \<comment> \<open>Suggested by Pierre Chartier\<close>
   by blast