src/ZF/Constructible/Reflection.thy
changeset 21232 faacfd4392b5
parent 16417 9bc16273c2d4
child 23464 bc2563c37b1a
--- a/src/ZF/Constructible/Reflection.thy	Tue Nov 07 19:39:53 2006 +0100
+++ b/src/ZF/Constructible/Reflection.thy	Tue Nov 07 19:39:54 2006 +0100
@@ -199,7 +199,7 @@
      "(!!a. [| Cl(a); Ord(a) |] ==> \<forall>x\<in>Mset(a). P(x) <-> Q(a,x))
       ==> Closed_Unbounded(ClEx(P))"
 apply (unfold ClEx_eq FF_def F0_def M_def) 
-apply (rule Reflection.ZF_Closed_Unbounded_ClEx [of Mset _ _ Cl])
+apply (rule ex_reflection.ZF_Closed_Unbounded_ClEx [of Mset _ _ Cl])
 apply (rule ex_reflection.intro, assumption)
 apply (blast intro: ex_reflection_axioms.intro)
 done