src/ZF/Constructible/Rec_Separation.thy
changeset 30729 461ee3e49ad3
parent 29223 e09c53289830
child 46823 57bf0cecb366
equal deleted inserted replaced
30728:f0aeca99b5d9 30729:461ee3e49ad3
   183   done
   183   done
   184 
   184 
   185 theorem M_trancl_L: "PROP M_trancl(L)"
   185 theorem M_trancl_L: "PROP M_trancl(L)"
   186 by (rule M_trancl.intro [OF M_basic_L M_trancl_axioms_L])
   186 by (rule M_trancl.intro [OF M_basic_L M_trancl_axioms_L])
   187 
   187 
   188 interpretation L: M_trancl L by (rule M_trancl_L)
   188 interpretation L?: M_trancl L by (rule M_trancl_L)
   189 
   189 
   190 
   190 
   191 subsection{*@{term L} is Closed Under the Operator @{term list}*}
   191 subsection{*@{term L} is Closed Under the Operator @{term list}*}
   192 
   192 
   193 subsubsection{*Instances of Replacement for Lists*}
   193 subsubsection{*Instances of Replacement for Lists*}
   370   apply (rule M_datatypes.intro)
   370   apply (rule M_datatypes.intro)
   371    apply (rule M_trancl_L)
   371    apply (rule M_trancl_L)
   372   apply (rule M_datatypes_axioms_L) 
   372   apply (rule M_datatypes_axioms_L) 
   373   done
   373   done
   374 
   374 
   375 interpretation L: M_datatypes L by (rule M_datatypes_L)
   375 interpretation L?: M_datatypes L by (rule M_datatypes_L)
   376 
   376 
   377 
   377 
   378 subsection{*@{term L} is Closed Under the Operator @{term eclose}*}
   378 subsection{*@{term L} is Closed Under the Operator @{term eclose}*}
   379 
   379 
   380 subsubsection{*Instances of Replacement for @{term eclose}*}
   380 subsubsection{*Instances of Replacement for @{term eclose}*}
   433   apply (rule M_eclose.intro)
   433   apply (rule M_eclose.intro)
   434    apply (rule M_datatypes_L)
   434    apply (rule M_datatypes_L)
   435   apply (rule M_eclose_axioms_L)
   435   apply (rule M_eclose_axioms_L)
   436   done
   436   done
   437 
   437 
   438 interpretation L: M_eclose L by (rule M_eclose_L)
   438 interpretation L?: M_eclose L by (rule M_eclose_L)
   439 
   439 
   440 
   440 
   441 end
   441 end