src/ZF/Constructible/L_axioms.thy
changeset 13434 78b93a667c01
parent 13429 2232810416fc
child 13440 cdde97e1db1c
--- a/src/ZF/Constructible/L_axioms.thy	Tue Jul 30 11:38:33 2002 +0200
+++ b/src/ZF/Constructible/L_axioms.thy	Tue Jul 30 11:39:57 2002 +0200
@@ -248,15 +248,17 @@
 done
 
 
+lemma reflection_Lset: "reflection(Lset)"
+apply (blast intro: reflection.intro Lset_mono_le Lset_cont Pair_in_Lset) +
+done
+
 theorem Ex_reflection:
      "REFLECTS[\<lambda>x. P(fst(x),snd(x)), \<lambda>a x. Q(a,fst(x),snd(x))]
       ==> REFLECTS[\<lambda>x. \<exists>z. L(z) \<and> P(x,z), \<lambda>a x. \<exists>z\<in>Lset(a). Q(a,x,z)]"
 apply (unfold L_Reflects_def L_ClEx_def L_FF_def L_F0_def L_def)
 apply (elim meta_exE)
 apply (rule meta_exI)
-apply (rule reflection.Ex_reflection
-  [OF reflection.intro, OF Lset_mono_le Lset_cont Pair_in_Lset],
-  assumption+)
+apply (erule reflection.Ex_reflection [OF reflection_Lset])
 done
 
 theorem All_reflection:
@@ -265,9 +267,7 @@
 apply (unfold L_Reflects_def L_ClEx_def L_FF_def L_F0_def L_def)
 apply (elim meta_exE)
 apply (rule meta_exI)
-apply (rule reflection.All_reflection
-  [OF reflection.intro, OF Lset_mono_le Lset_cont Pair_in_Lset],
-       assumption+)
+apply (erule reflection.All_reflection [OF reflection_Lset])
 done
 
 theorem Rex_reflection: