src/ZF/Constructible/Rec_Separation.thy
changeset 19931 fb32b43e7f80
parent 16417 9bc16273c2d4
child 21233 5a5c8ea5f66a
equal deleted inserted replaced
19930:baeb0aeb4891 19931:fb32b43e7f80
   179   apply (rule M_trancl_axioms.intro)
   179   apply (rule M_trancl_axioms.intro)
   180    apply (assumption | rule rtrancl_separation wellfounded_trancl_separation)+
   180    apply (assumption | rule rtrancl_separation wellfounded_trancl_separation)+
   181   done
   181   done
   182 
   182 
   183 theorem M_trancl_L: "PROP M_trancl(L)"
   183 theorem M_trancl_L: "PROP M_trancl(L)"
   184 by (rule M_trancl.intro
   184 by (rule M_trancl.intro [OF M_basic_L M_trancl_axioms_L])
   185          [OF M_trivial_L M_basic_axioms_L M_trancl_axioms_L])
   185 
   186 
   186 interpretation M_trancl [L] by (rule M_trancl_L)
   187 interpretation M_trancl [L] by (rule M_trancl_axioms_L)
       
   188 
   187 
   189 
   188 
   190 subsection{*@{term L} is Closed Under the Operator @{term list}*}
   189 subsection{*@{term L} is Closed Under the Operator @{term list}*}
   191 
   190 
   192 subsubsection{*Instances of Replacement for Lists*}
   191 subsubsection{*Instances of Replacement for Lists*}
   364         nth_replacement)+
   363         nth_replacement)+
   365   done
   364   done
   366 
   365 
   367 theorem M_datatypes_L: "PROP M_datatypes(L)"
   366 theorem M_datatypes_L: "PROP M_datatypes(L)"
   368   apply (rule M_datatypes.intro)
   367   apply (rule M_datatypes.intro)
   369       apply (rule M_trancl.axioms [OF M_trancl_L])+
   368    apply (rule M_trancl_L)
   370  apply (rule M_datatypes_axioms_L) 
   369   apply (rule M_datatypes_axioms_L) 
   371  done
   370   done
   372 
   371 
   373 interpretation M_datatypes [L] by (rule M_datatypes_axioms_L)
   372 interpretation M_datatypes [L] by (rule M_datatypes_L)
   374 
   373 
   375 
   374 
   376 subsection{*@{term L} is Closed Under the Operator @{term eclose}*}
   375 subsection{*@{term L} is Closed Under the Operator @{term eclose}*}
   377 
   376 
   378 subsubsection{*Instances of Replacement for @{term eclose}*}
   377 subsubsection{*Instances of Replacement for @{term eclose}*}
   427    apply (assumption | rule eclose_replacement1 eclose_replacement2)+
   426    apply (assumption | rule eclose_replacement1 eclose_replacement2)+
   428   done
   427   done
   429 
   428 
   430 theorem M_eclose_L: "PROP M_eclose(L)"
   429 theorem M_eclose_L: "PROP M_eclose(L)"
   431   apply (rule M_eclose.intro)
   430   apply (rule M_eclose.intro)
   432        apply (rule M_datatypes.axioms [OF M_datatypes_L])+
   431    apply (rule M_datatypes_L)
   433   apply (rule M_eclose_axioms_L)
   432   apply (rule M_eclose_axioms_L)
   434   done
   433   done
   435 
   434 
   436 interpretation M_eclose [L] by (rule M_eclose_axioms_L)
   435 interpretation M_eclose [L] by (rule M_eclose_L)
   437 
   436 
   438 
   437 
   439 end
   438 end