src/ZF/Constructible/Reflection.thy
changeset 23464 bc2563c37b1a
parent 21232 faacfd4392b5
child 32960 69916a850301
--- a/src/ZF/Constructible/Reflection.thy	Thu Jun 21 17:28:53 2007 +0200
+++ b/src/ZF/Constructible/Reflection.thy	Thu Jun 21 20:07:26 2007 +0200
@@ -200,7 +200,7 @@
       ==> Closed_Unbounded(ClEx(P))"
 apply (unfold ClEx_eq FF_def F0_def M_def) 
 apply (rule ex_reflection.ZF_Closed_Unbounded_ClEx [of Mset _ _ Cl])
-apply (rule ex_reflection.intro, assumption)
+apply (rule ex_reflection.intro, rule reflection_axioms)
 apply (blast intro: ex_reflection_axioms.intro)
 done