src/ZF/Constructible/Rec_Separation.thy
changeset 13506 acc18a5d2b1a
parent 13505 52a16cb7fefb
child 13564 1500a2e48d44
equal deleted inserted replaced
13505:52a16cb7fefb 13506:acc18a5d2b1a
   170 apply (intro FOL_reflections function_reflections
   170 apply (intro FOL_reflections function_reflections
   171              rtran_closure_reflection composition_reflection)
   171              rtran_closure_reflection composition_reflection)
   172 done
   172 done
   173 
   173 
   174 
   174 
   175 subsection{*Separation for the Proof of @{text "wellfounded_on_trancl"}*}
   175 subsubsection{*Separation for the Proof of @{text "wellfounded_on_trancl"}*}
   176 
   176 
   177 lemma wellfounded_trancl_reflects:
   177 lemma wellfounded_trancl_reflects:
   178   "REFLECTS[\<lambda>x. \<exists>w[L]. \<exists>wx[L]. \<exists>rp[L].
   178   "REFLECTS[\<lambda>x. \<exists>w[L]. \<exists>wx[L]. \<exists>rp[L].
   179                  w \<in> Z & pair(L,w,x,wx) & tran_closure(L,r,rp) & wx \<in> rp,
   179                  w \<in> Z & pair(L,w,x,wx) & tran_closure(L,r,rp) & wx \<in> rp,
   180    \<lambda>i x. \<exists>w \<in> Lset(i). \<exists>wx \<in> Lset(i). \<exists>rp \<in> Lset(i).
   180    \<lambda>i x. \<exists>w \<in> Lset(i). \<exists>wx \<in> Lset(i). \<exists>rp \<in> Lset(i).