src/HOL/UNITY/ProgressSets.thy
changeset 32139 e271a64f03ff
parent 30198 922f944f03b2
child 32604 8b3e2bc91a46
--- a/src/HOL/UNITY/ProgressSets.thy	Wed Jul 22 14:21:52 2009 +0200
+++ b/src/HOL/UNITY/ProgressSets.thy	Wed Jul 22 18:02:10 2009 +0200
@@ -44,7 +44,7 @@
 
 lemma UN_in_lattice:
      "[|lattice L; !!i. i\<in>I ==> r i \<in> L|] ==> (\<Union>i\<in>I. r i) \<in> L"
-apply (simp add: Set.UN_eq) 
+apply (simp add: UN_eq) 
 apply (blast intro: Union_in_lattice) 
 done