src/HOL/Analysis/Starlike.thy
changeset 69313 b021008c5397
parent 69286 e4d5a07fecb6
child 69325 4b6ddc5989fc
--- a/src/HOL/Analysis/Starlike.thy	Sun Nov 18 09:51:41 2018 +0100
+++ b/src/HOL/Analysis/Starlike.thy	Sun Nov 18 18:07:51 2018 +0000
@@ -7494,9 +7494,9 @@
                     and clos: "closure (G x) \<subseteq> F x" and Fin: "F x \<in> \<C>"
          if "x \<in> S" for x
     by metis
-  then obtain \<F> where "\<F> \<subseteq> G ` S" "countable \<F>" "\<Union>\<F> = UNION S G"
+  then obtain \<F> where "\<F> \<subseteq> G ` S" "countable \<F>" "\<Union>\<F> = \<Union>(G ` S)"
     using Lindelof [of "G ` S"] by (metis image_iff)
-  then obtain K where K: "K \<subseteq> S" "countable K" and eq: "UNION K G = UNION S G"
+  then obtain K where K: "K \<subseteq> S" "countable K" and eq: "\<Union>(G ` K) = \<Union>(G ` S)"
     by (metis countable_subset_image)
   with False Gin have "K \<noteq> {}" by force
   then obtain a :: "nat \<Rightarrow> 'a" where "range a = K"
@@ -7885,7 +7885,7 @@
     obtain I where "finite I" and I: "K \<subseteq> (\<Union>i\<in>I. interior (f i))"
     proof (rule compactE_image [OF \<open>compact K\<close>])
       show "K \<subseteq> (\<Union>n. interior (f n))"
-        using \<open>K \<subseteq> S\<close> \<open>UNION UNIV f = S\<close> * by blast
+        using \<open>K \<subseteq> S\<close> \<open>\<Union>(f ` UNIV) = S\<close> * by blast
     qed auto
     { fix n
       assume n: "Max I \<le> n"