dropped errorneous hint
authorhaftmann
Fri, 22 Jul 2011 07:33:29 +0200
changeset 43944 b1b436f75070
parent 43943 e6928fc2332a
child 43945 48065e997df0
dropped errorneous hint
src/HOL/Complete_Lattice.thy
--- a/src/HOL/Complete_Lattice.thy	Thu Jul 21 22:47:13 2011 +0200
+++ b/src/HOL/Complete_Lattice.thy	Fri Jul 22 07:33:29 2011 +0200
@@ -941,7 +941,7 @@
 lemma UN_eq: "(\<Union>x\<in>A. B x) = \<Union>({Y. \<exists>x\<in>A. Y = B x})"
   by (fact SUP_eq)
 
-lemma image_Union: "f ` \<Union>S = (\<Union>x\<in>S. f ` x)" -- "FIXME generalize"
+lemma image_Union: "f ` \<Union>S = (\<Union>x\<in>S. f ` x)"
   by blast
 
 lemma UNION_empty_conv[simp]: