src/ZF/Constructible/Separation.thy
changeset 13428 99e52e78eb65
parent 13385 31df66ca0780
child 13429 2232810416fc
equal deleted inserted replaced
13427:b429fd98549c 13428:99e52e78eb65
     7 text{*Helps us solve for de Bruijn indices!*}
     7 text{*Helps us solve for de Bruijn indices!*}
     8 lemma nth_ConsI: "[|nth(n,l) = x; n \<in> nat|] ==> nth(succ(n), Cons(a,l)) = x"
     8 lemma nth_ConsI: "[|nth(n,l) = x; n \<in> nat|] ==> nth(succ(n), Cons(a,l)) = x"
     9 by simp
     9 by simp
    10 
    10 
    11 lemmas nth_rules = nth_0 nth_ConsI nat_0I nat_succI
    11 lemmas nth_rules = nth_0 nth_ConsI nat_0I nat_succI
    12 lemmas sep_rules = nth_0 nth_ConsI FOL_iff_sats function_iff_sats 
    12 lemmas sep_rules = nth_0 nth_ConsI FOL_iff_sats function_iff_sats
    13                    fun_plus_iff_sats
    13                    fun_plus_iff_sats
    14 
    14 
    15 lemma Collect_conj_in_DPow:
    15 lemma Collect_conj_in_DPow:
    16      "[| {x\<in>A. P(x)} \<in> DPow(A);  {x\<in>A. Q(x)} \<in> DPow(A) |] 
    16      "[| {x\<in>A. P(x)} \<in> DPow(A);  {x\<in>A. Q(x)} \<in> DPow(A) |]
    17       ==> {x\<in>A. P(x) & Q(x)} \<in> DPow(A)"
    17       ==> {x\<in>A. P(x) & Q(x)} \<in> DPow(A)"
    18 by (simp add: Int_in_DPow Collect_Int_Collect_eq [symmetric]) 
    18 by (simp add: Int_in_DPow Collect_Int_Collect_eq [symmetric])
    19 
    19 
    20 lemma Collect_conj_in_DPow_Lset:
    20 lemma Collect_conj_in_DPow_Lset:
    21      "[|z \<in> Lset(j); {x \<in> Lset(j). P(x)} \<in> DPow(Lset(j))|]
    21      "[|z \<in> Lset(j); {x \<in> Lset(j). P(x)} \<in> DPow(Lset(j))|]
    22       ==> {x \<in> Lset(j). x \<in> z & P(x)} \<in> DPow(Lset(j))"
    22       ==> {x \<in> Lset(j). x \<in> z & P(x)} \<in> DPow(Lset(j))"
    23 apply (frule mem_Lset_imp_subset_Lset)
    23 apply (frule mem_Lset_imp_subset_Lset)
    24 apply (simp add: Collect_conj_in_DPow Collect_mem_eq 
    24 apply (simp add: Collect_conj_in_DPow Collect_mem_eq
    25                  subset_Int_iff2 elem_subset_in_DPow)
    25                  subset_Int_iff2 elem_subset_in_DPow)
    26 done
    26 done
    27 
    27 
    28 lemma separation_CollectI:
    28 lemma separation_CollectI:
    29      "(\<And>z. L(z) ==> L({x \<in> z . P(x)})) ==> separation(L, \<lambda>x. P(x))"
    29      "(\<And>z. L(z) ==> L({x \<in> z . P(x)})) ==> separation(L, \<lambda>x. P(x))"
    30 apply (unfold separation_def, clarify) 
    30 apply (unfold separation_def, clarify)
    31 apply (rule_tac x="{x\<in>z. P(x)}" in rexI) 
    31 apply (rule_tac x="{x\<in>z. P(x)}" in rexI)
    32 apply simp_all
    32 apply simp_all
    33 done
    33 done
    34 
    34 
    35 text{*Reduces the original comprehension to the reflected one*}
    35 text{*Reduces the original comprehension to the reflected one*}
    36 lemma reflection_imp_L_separation:
    36 lemma reflection_imp_L_separation:
    37       "[| \<forall>x\<in>Lset(j). P(x) <-> Q(x);
    37       "[| \<forall>x\<in>Lset(j). P(x) <-> Q(x);
    38           {x \<in> Lset(j) . Q(x)} \<in> DPow(Lset(j)); 
    38           {x \<in> Lset(j) . Q(x)} \<in> DPow(Lset(j));
    39           Ord(j);  z \<in> Lset(j)|] ==> L({x \<in> z . P(x)})"
    39           Ord(j);  z \<in> Lset(j)|] ==> L({x \<in> z . P(x)})"
    40 apply (rule_tac i = "succ(j)" in L_I)
    40 apply (rule_tac i = "succ(j)" in L_I)
    41  prefer 2 apply simp
    41  prefer 2 apply simp
    42 apply (subgoal_tac "{x \<in> z. P(x)} = {x \<in> Lset(j). x \<in> z & (Q(x))}")
    42 apply (subgoal_tac "{x \<in> z. P(x)} = {x \<in> Lset(j). x \<in> z & (Q(x))}")
    43  prefer 2
    43  prefer 2
    44  apply (blast dest: mem_Lset_imp_subset_Lset) 
    44  apply (blast dest: mem_Lset_imp_subset_Lset)
    45 apply (simp add: Lset_succ Collect_conj_in_DPow_Lset)
    45 apply (simp add: Lset_succ Collect_conj_in_DPow_Lset)
    46 done
    46 done
    47 
    47 
    48 
    48 
    49 subsection{*Separation for Intersection*}
    49 subsection{*Separation for Intersection*}
    50 
    50 
    51 lemma Inter_Reflects:
    51 lemma Inter_Reflects:
    52      "REFLECTS[\<lambda>x. \<forall>y[L]. y\<in>A --> x \<in> y, 
    52      "REFLECTS[\<lambda>x. \<forall>y[L]. y\<in>A --> x \<in> y,
    53                \<lambda>i x. \<forall>y\<in>Lset(i). y\<in>A --> x \<in> y]"
    53                \<lambda>i x. \<forall>y\<in>Lset(i). y\<in>A --> x \<in> y]"
    54 by (intro FOL_reflections)  
    54 by (intro FOL_reflections)
    55 
    55 
    56 lemma Inter_separation:
    56 lemma Inter_separation:
    57      "L(A) ==> separation(L, \<lambda>x. \<forall>y[L]. y\<in>A --> x\<in>y)"
    57      "L(A) ==> separation(L, \<lambda>x. \<forall>y[L]. y\<in>A --> x\<in>y)"
    58 apply (rule separation_CollectI) 
    58 apply (rule separation_CollectI)
    59 apply (rule_tac A="{A,z}" in subset_LsetE, blast ) 
    59 apply (rule_tac A="{A,z}" in subset_LsetE, blast )
    60 apply (rule ReflectsE [OF Inter_Reflects], assumption)
    60 apply (rule ReflectsE [OF Inter_Reflects], assumption)
    61 apply (drule subset_Lset_ltD, assumption) 
    61 apply (drule subset_Lset_ltD, assumption)
    62 apply (erule reflection_imp_L_separation)
    62 apply (erule reflection_imp_L_separation)
    63   apply (simp_all add: lt_Ord2, clarify)
    63   apply (simp_all add: lt_Ord2, clarify)
    64 apply (rule DPow_LsetI) 
    64 apply (rule DPow_LsetI)
    65 apply (rule ball_iff_sats) 
    65 apply (rule ball_iff_sats)
    66 apply (rule imp_iff_sats)
    66 apply (rule imp_iff_sats)
    67 apply (rule_tac [2] i=1 and j=0 and env="[y,x,A]" in mem_iff_sats)
    67 apply (rule_tac [2] i=1 and j=0 and env="[y,x,A]" in mem_iff_sats)
    68 apply (rule_tac i=0 and j=2 in mem_iff_sats)
    68 apply (rule_tac i=0 and j=2 in mem_iff_sats)
    69 apply (simp_all add: succ_Un_distrib [symmetric])
    69 apply (simp_all add: succ_Un_distrib [symmetric])
    70 done
    70 done
    71 
    71 
    72 subsection{*Separation for Cartesian Product*}
    72 subsection{*Separation for Cartesian Product*}
    73 
    73 
    74 lemma cartprod_Reflects:
    74 lemma cartprod_Reflects:
    75      "REFLECTS[\<lambda>z. \<exists>x[L]. x\<in>A & (\<exists>y[L]. y\<in>B & pair(L,x,y,z)),
    75      "REFLECTS[\<lambda>z. \<exists>x[L]. x\<in>A & (\<exists>y[L]. y\<in>B & pair(L,x,y,z)),
    76                 \<lambda>i z. \<exists>x\<in>Lset(i). x\<in>A & (\<exists>y\<in>Lset(i). y\<in>B & 
    76                 \<lambda>i z. \<exists>x\<in>Lset(i). x\<in>A & (\<exists>y\<in>Lset(i). y\<in>B &
    77                                    pair(**Lset(i),x,y,z))]"
    77                                    pair(**Lset(i),x,y,z))]"
    78 by (intro FOL_reflections function_reflections)
    78 by (intro FOL_reflections function_reflections)
    79 
    79 
    80 lemma cartprod_separation:
    80 lemma cartprod_separation:
    81      "[| L(A); L(B) |] 
    81      "[| L(A); L(B) |]
    82       ==> separation(L, \<lambda>z. \<exists>x[L]. x\<in>A & (\<exists>y[L]. y\<in>B & pair(L,x,y,z)))"
    82       ==> separation(L, \<lambda>z. \<exists>x[L]. x\<in>A & (\<exists>y[L]. y\<in>B & pair(L,x,y,z)))"
    83 apply (rule separation_CollectI) 
    83 apply (rule separation_CollectI)
    84 apply (rule_tac A="{A,B,z}" in subset_LsetE, blast ) 
    84 apply (rule_tac A="{A,B,z}" in subset_LsetE, blast )
    85 apply (rule ReflectsE [OF cartprod_Reflects], assumption)
    85 apply (rule ReflectsE [OF cartprod_Reflects], assumption)
    86 apply (drule subset_Lset_ltD, assumption) 
    86 apply (drule subset_Lset_ltD, assumption)
    87 apply (erule reflection_imp_L_separation)
    87 apply (erule reflection_imp_L_separation)
    88   apply (simp_all add: lt_Ord2, clarify) 
    88   apply (simp_all add: lt_Ord2, clarify)
    89 apply (rule DPow_LsetI)
    89 apply (rule DPow_LsetI)
    90 apply (rename_tac u)  
    90 apply (rename_tac u)
    91 apply (rule bex_iff_sats) 
    91 apply (rule bex_iff_sats)
    92 apply (rule conj_iff_sats)
    92 apply (rule conj_iff_sats)
    93 apply (rule_tac i=0 and j=2 and env="[x,u,A,B]" in mem_iff_sats, simp_all)
    93 apply (rule_tac i=0 and j=2 and env="[x,u,A,B]" in mem_iff_sats, simp_all)
    94 apply (rule sep_rules | simp)+
    94 apply (rule sep_rules | simp)+
    95 done
    95 done
    96 
    96 
   100      "REFLECTS[\<lambda>y. \<exists>p[L]. p\<in>r & (\<exists>x[L]. x\<in>A & pair(L,x,y,p)),
   100      "REFLECTS[\<lambda>y. \<exists>p[L]. p\<in>r & (\<exists>x[L]. x\<in>A & pair(L,x,y,p)),
   101            \<lambda>i y. \<exists>p\<in>Lset(i). p\<in>r & (\<exists>x\<in>Lset(i). x\<in>A & pair(**Lset(i),x,y,p))]"
   101            \<lambda>i y. \<exists>p\<in>Lset(i). p\<in>r & (\<exists>x\<in>Lset(i). x\<in>A & pair(**Lset(i),x,y,p))]"
   102 by (intro FOL_reflections function_reflections)
   102 by (intro FOL_reflections function_reflections)
   103 
   103 
   104 lemma image_separation:
   104 lemma image_separation:
   105      "[| L(A); L(r) |] 
   105      "[| L(A); L(r) |]
   106       ==> separation(L, \<lambda>y. \<exists>p[L]. p\<in>r & (\<exists>x[L]. x\<in>A & pair(L,x,y,p)))"
   106       ==> separation(L, \<lambda>y. \<exists>p[L]. p\<in>r & (\<exists>x[L]. x\<in>A & pair(L,x,y,p)))"
   107 apply (rule separation_CollectI) 
   107 apply (rule separation_CollectI)
   108 apply (rule_tac A="{A,r,z}" in subset_LsetE, blast ) 
   108 apply (rule_tac A="{A,r,z}" in subset_LsetE, blast )
   109 apply (rule ReflectsE [OF image_Reflects], assumption)
   109 apply (rule ReflectsE [OF image_Reflects], assumption)
   110 apply (drule subset_Lset_ltD, assumption) 
   110 apply (drule subset_Lset_ltD, assumption)
   111 apply (erule reflection_imp_L_separation)
   111 apply (erule reflection_imp_L_separation)
   112   apply (simp_all add: lt_Ord2, clarify)
   112   apply (simp_all add: lt_Ord2, clarify)
   113 apply (rule DPow_LsetI)
   113 apply (rule DPow_LsetI)
   114 apply (rule bex_iff_sats) 
   114 apply (rule bex_iff_sats)
   115 apply (rule conj_iff_sats)
   115 apply (rule conj_iff_sats)
   116 apply (rule_tac env="[p,y,A,r]" in mem_iff_sats)
   116 apply (rule_tac env="[p,y,A,r]" in mem_iff_sats)
   117 apply (rule sep_rules | simp)+
   117 apply (rule sep_rules | simp)+
   118 done
   118 done
   119 
   119 
   120 
   120 
   121 subsection{*Separation for Converse*}
   121 subsection{*Separation for Converse*}
   122 
   122 
   123 lemma converse_Reflects:
   123 lemma converse_Reflects:
   124   "REFLECTS[\<lambda>z. \<exists>p[L]. p\<in>r & (\<exists>x[L]. \<exists>y[L]. pair(L,x,y,p) & pair(L,y,x,z)),
   124   "REFLECTS[\<lambda>z. \<exists>p[L]. p\<in>r & (\<exists>x[L]. \<exists>y[L]. pair(L,x,y,p) & pair(L,y,x,z)),
   125      \<lambda>i z. \<exists>p\<in>Lset(i). p\<in>r & (\<exists>x\<in>Lset(i). \<exists>y\<in>Lset(i). 
   125      \<lambda>i z. \<exists>p\<in>Lset(i). p\<in>r & (\<exists>x\<in>Lset(i). \<exists>y\<in>Lset(i).
   126                      pair(**Lset(i),x,y,p) & pair(**Lset(i),y,x,z))]"
   126                      pair(**Lset(i),x,y,p) & pair(**Lset(i),y,x,z))]"
   127 by (intro FOL_reflections function_reflections)
   127 by (intro FOL_reflections function_reflections)
   128 
   128 
   129 lemma converse_separation:
   129 lemma converse_separation:
   130      "L(r) ==> separation(L, 
   130      "L(r) ==> separation(L,
   131          \<lambda>z. \<exists>p[L]. p\<in>r & (\<exists>x[L]. \<exists>y[L]. pair(L,x,y,p) & pair(L,y,x,z)))"
   131          \<lambda>z. \<exists>p[L]. p\<in>r & (\<exists>x[L]. \<exists>y[L]. pair(L,x,y,p) & pair(L,y,x,z)))"
   132 apply (rule separation_CollectI) 
   132 apply (rule separation_CollectI)
   133 apply (rule_tac A="{r,z}" in subset_LsetE, blast ) 
   133 apply (rule_tac A="{r,z}" in subset_LsetE, blast )
   134 apply (rule ReflectsE [OF converse_Reflects], assumption)
   134 apply (rule ReflectsE [OF converse_Reflects], assumption)
   135 apply (drule subset_Lset_ltD, assumption) 
   135 apply (drule subset_Lset_ltD, assumption)
   136 apply (erule reflection_imp_L_separation)
   136 apply (erule reflection_imp_L_separation)
   137   apply (simp_all add: lt_Ord2, clarify)
   137   apply (simp_all add: lt_Ord2, clarify)
   138 apply (rule DPow_LsetI)
   138 apply (rule DPow_LsetI)
   139 apply (rename_tac u) 
   139 apply (rename_tac u)
   140 apply (rule bex_iff_sats) 
   140 apply (rule bex_iff_sats)
   141 apply (rule conj_iff_sats)
   141 apply (rule conj_iff_sats)
   142 apply (rule_tac i=0 and j=2 and env="[p,u,r]" in mem_iff_sats, simp_all)
   142 apply (rule_tac i=0 and j=2 and env="[p,u,r]" in mem_iff_sats, simp_all)
   143 apply (rule sep_rules | simp)+
   143 apply (rule sep_rules | simp)+
   144 done
   144 done
   145 
   145 
   151         \<lambda>i z. \<exists>x\<in>Lset(i). x\<in>A & (\<exists>y\<in>Lset(i). pair(**Lset(i),x,y,z))]"
   151         \<lambda>i z. \<exists>x\<in>Lset(i). x\<in>A & (\<exists>y\<in>Lset(i). pair(**Lset(i),x,y,z))]"
   152 by (intro FOL_reflections function_reflections)
   152 by (intro FOL_reflections function_reflections)
   153 
   153 
   154 lemma restrict_separation:
   154 lemma restrict_separation:
   155    "L(A) ==> separation(L, \<lambda>z. \<exists>x[L]. x\<in>A & (\<exists>y[L]. pair(L,x,y,z)))"
   155    "L(A) ==> separation(L, \<lambda>z. \<exists>x[L]. x\<in>A & (\<exists>y[L]. pair(L,x,y,z)))"
   156 apply (rule separation_CollectI) 
   156 apply (rule separation_CollectI)
   157 apply (rule_tac A="{A,z}" in subset_LsetE, blast ) 
   157 apply (rule_tac A="{A,z}" in subset_LsetE, blast )
   158 apply (rule ReflectsE [OF restrict_Reflects], assumption)
   158 apply (rule ReflectsE [OF restrict_Reflects], assumption)
   159 apply (drule subset_Lset_ltD, assumption) 
   159 apply (drule subset_Lset_ltD, assumption)
   160 apply (erule reflection_imp_L_separation)
   160 apply (erule reflection_imp_L_separation)
   161   apply (simp_all add: lt_Ord2, clarify)
   161   apply (simp_all add: lt_Ord2, clarify)
   162 apply (rule DPow_LsetI)
   162 apply (rule DPow_LsetI)
   163 apply (rename_tac u) 
   163 apply (rename_tac u)
   164 apply (rule bex_iff_sats) 
   164 apply (rule bex_iff_sats)
   165 apply (rule conj_iff_sats)
   165 apply (rule conj_iff_sats)
   166 apply (rule_tac i=0 and j=2 and env="[x,u,A]" in mem_iff_sats, simp_all)
   166 apply (rule_tac i=0 and j=2 and env="[x,u,A]" in mem_iff_sats, simp_all)
   167 apply (rule sep_rules | simp)+
   167 apply (rule sep_rules | simp)+
   168 done
   168 done
   169 
   169 
   170 
   170 
   171 subsection{*Separation for Composition*}
   171 subsection{*Separation for Composition*}
   172 
   172 
   173 lemma comp_Reflects:
   173 lemma comp_Reflects:
   174      "REFLECTS[\<lambda>xz. \<exists>x[L]. \<exists>y[L]. \<exists>z[L]. \<exists>xy[L]. \<exists>yz[L]. 
   174      "REFLECTS[\<lambda>xz. \<exists>x[L]. \<exists>y[L]. \<exists>z[L]. \<exists>xy[L]. \<exists>yz[L].
   175 		  pair(L,x,z,xz) & pair(L,x,y,xy) & pair(L,y,z,yz) & 
   175                   pair(L,x,z,xz) & pair(L,x,y,xy) & pair(L,y,z,yz) &
   176                   xy\<in>s & yz\<in>r,
   176                   xy\<in>s & yz\<in>r,
   177         \<lambda>i xz. \<exists>x\<in>Lset(i). \<exists>y\<in>Lset(i). \<exists>z\<in>Lset(i). \<exists>xy\<in>Lset(i). \<exists>yz\<in>Lset(i). 
   177         \<lambda>i xz. \<exists>x\<in>Lset(i). \<exists>y\<in>Lset(i). \<exists>z\<in>Lset(i). \<exists>xy\<in>Lset(i). \<exists>yz\<in>Lset(i).
   178 		  pair(**Lset(i),x,z,xz) & pair(**Lset(i),x,y,xy) & 
   178                   pair(**Lset(i),x,z,xz) & pair(**Lset(i),x,y,xy) &
   179                   pair(**Lset(i),y,z,yz) & xy\<in>s & yz\<in>r]"
   179                   pair(**Lset(i),y,z,yz) & xy\<in>s & yz\<in>r]"
   180 by (intro FOL_reflections function_reflections)
   180 by (intro FOL_reflections function_reflections)
   181 
   181 
   182 lemma comp_separation:
   182 lemma comp_separation:
   183      "[| L(r); L(s) |]
   183      "[| L(r); L(s) |]
   184       ==> separation(L, \<lambda>xz. \<exists>x[L]. \<exists>y[L]. \<exists>z[L]. \<exists>xy[L]. \<exists>yz[L]. 
   184       ==> separation(L, \<lambda>xz. \<exists>x[L]. \<exists>y[L]. \<exists>z[L]. \<exists>xy[L]. \<exists>yz[L].
   185 		  pair(L,x,z,xz) & pair(L,x,y,xy) & pair(L,y,z,yz) & 
   185                   pair(L,x,z,xz) & pair(L,x,y,xy) & pair(L,y,z,yz) &
   186                   xy\<in>s & yz\<in>r)"
   186                   xy\<in>s & yz\<in>r)"
   187 apply (rule separation_CollectI) 
   187 apply (rule separation_CollectI)
   188 apply (rule_tac A="{r,s,z}" in subset_LsetE, blast ) 
   188 apply (rule_tac A="{r,s,z}" in subset_LsetE, blast )
   189 apply (rule ReflectsE [OF comp_Reflects], assumption)
   189 apply (rule ReflectsE [OF comp_Reflects], assumption)
   190 apply (drule subset_Lset_ltD, assumption) 
   190 apply (drule subset_Lset_ltD, assumption)
   191 apply (erule reflection_imp_L_separation)
   191 apply (erule reflection_imp_L_separation)
   192   apply (simp_all add: lt_Ord2, clarify)
   192   apply (simp_all add: lt_Ord2, clarify)
   193 apply (rule DPow_LsetI)
   193 apply (rule DPow_LsetI)
   194 apply (rename_tac u) 
   194 apply (rename_tac u)
   195 apply (rule bex_iff_sats)+
   195 apply (rule bex_iff_sats)+
   196 apply (rename_tac x y z)  
   196 apply (rename_tac x y z)
   197 apply (rule conj_iff_sats)
   197 apply (rule conj_iff_sats)
   198 apply (rule_tac env="[z,y,x,u,r,s]" in pair_iff_sats)
   198 apply (rule_tac env="[z,y,x,u,r,s]" in pair_iff_sats)
   199 apply (rule sep_rules | simp)+
   199 apply (rule sep_rules | simp)+
   200 done
   200 done
   201 
   201 
   206                     \<lambda>i y. \<exists>p \<in> Lset(i). p\<in>r & pair(**Lset(i),y,x,p)]"
   206                     \<lambda>i y. \<exists>p \<in> Lset(i). p\<in>r & pair(**Lset(i),y,x,p)]"
   207 by (intro FOL_reflections function_reflections)
   207 by (intro FOL_reflections function_reflections)
   208 
   208 
   209 lemma pred_separation:
   209 lemma pred_separation:
   210      "[| L(r); L(x) |] ==> separation(L, \<lambda>y. \<exists>p[L]. p\<in>r & pair(L,y,x,p))"
   210      "[| L(r); L(x) |] ==> separation(L, \<lambda>y. \<exists>p[L]. p\<in>r & pair(L,y,x,p))"
   211 apply (rule separation_CollectI) 
   211 apply (rule separation_CollectI)
   212 apply (rule_tac A="{r,x,z}" in subset_LsetE, blast ) 
   212 apply (rule_tac A="{r,x,z}" in subset_LsetE, blast )
   213 apply (rule ReflectsE [OF pred_Reflects], assumption)
   213 apply (rule ReflectsE [OF pred_Reflects], assumption)
   214 apply (drule subset_Lset_ltD, assumption) 
   214 apply (drule subset_Lset_ltD, assumption)
   215 apply (erule reflection_imp_L_separation)
   215 apply (erule reflection_imp_L_separation)
   216   apply (simp_all add: lt_Ord2, clarify)
   216   apply (simp_all add: lt_Ord2, clarify)
   217 apply (rule DPow_LsetI)
   217 apply (rule DPow_LsetI)
   218 apply (rename_tac u) 
   218 apply (rename_tac u)
   219 apply (rule bex_iff_sats)
   219 apply (rule bex_iff_sats)
   220 apply (rule conj_iff_sats)
   220 apply (rule conj_iff_sats)
   221 apply (rule_tac env = "[p,u,r,x]" in mem_iff_sats) 
   221 apply (rule_tac env = "[p,u,r,x]" in mem_iff_sats)
   222 apply (rule sep_rules | simp)+
   222 apply (rule sep_rules | simp)+
   223 done
   223 done
   224 
   224 
   225 
   225 
   226 subsection{*Separation for the Membership Relation*}
   226 subsection{*Separation for the Membership Relation*}
   230             \<lambda>i z. \<exists>x \<in> Lset(i). \<exists>y \<in> Lset(i). pair(**Lset(i),x,y,z) & x \<in> y]"
   230             \<lambda>i z. \<exists>x \<in> Lset(i). \<exists>y \<in> Lset(i). pair(**Lset(i),x,y,z) & x \<in> y]"
   231 by (intro FOL_reflections function_reflections)
   231 by (intro FOL_reflections function_reflections)
   232 
   232 
   233 lemma Memrel_separation:
   233 lemma Memrel_separation:
   234      "separation(L, \<lambda>z. \<exists>x[L]. \<exists>y[L]. pair(L,x,y,z) & x \<in> y)"
   234      "separation(L, \<lambda>z. \<exists>x[L]. \<exists>y[L]. pair(L,x,y,z) & x \<in> y)"
   235 apply (rule separation_CollectI) 
   235 apply (rule separation_CollectI)
   236 apply (rule_tac A="{z}" in subset_LsetE, blast ) 
   236 apply (rule_tac A="{z}" in subset_LsetE, blast )
   237 apply (rule ReflectsE [OF Memrel_Reflects], assumption)
   237 apply (rule ReflectsE [OF Memrel_Reflects], assumption)
   238 apply (drule subset_Lset_ltD, assumption) 
   238 apply (drule subset_Lset_ltD, assumption)
   239 apply (erule reflection_imp_L_separation)
   239 apply (erule reflection_imp_L_separation)
   240   apply (simp_all add: lt_Ord2)
   240   apply (simp_all add: lt_Ord2)
   241 apply (rule DPow_LsetI)
   241 apply (rule DPow_LsetI)
   242 apply (rename_tac u) 
   242 apply (rename_tac u)
   243 apply (rule bex_iff_sats conj_iff_sats)+
   243 apply (rule bex_iff_sats conj_iff_sats)+
   244 apply (rule_tac env = "[y,x,u]" in pair_iff_sats) 
   244 apply (rule_tac env = "[y,x,u]" in pair_iff_sats)
   245 apply (rule sep_rules | simp)+
   245 apply (rule sep_rules | simp)+
   246 done
   246 done
   247 
   247 
   248 
   248 
   249 subsection{*Replacement for FunSpace*}
   249 subsection{*Replacement for FunSpace*}
   250 		
   250 
   251 lemma funspace_succ_Reflects:
   251 lemma funspace_succ_Reflects:
   252  "REFLECTS[\<lambda>z. \<exists>p[L]. p\<in>A & (\<exists>f[L]. \<exists>b[L]. \<exists>nb[L]. \<exists>cnbf[L]. 
   252  "REFLECTS[\<lambda>z. \<exists>p[L]. p\<in>A & (\<exists>f[L]. \<exists>b[L]. \<exists>nb[L]. \<exists>cnbf[L].
   253 	    pair(L,f,b,p) & pair(L,n,b,nb) & is_cons(L,nb,f,cnbf) &
   253             pair(L,f,b,p) & pair(L,n,b,nb) & is_cons(L,nb,f,cnbf) &
   254 	    upair(L,cnbf,cnbf,z)),
   254             upair(L,cnbf,cnbf,z)),
   255 	\<lambda>i z. \<exists>p \<in> Lset(i). p\<in>A & (\<exists>f \<in> Lset(i). \<exists>b \<in> Lset(i). 
   255         \<lambda>i z. \<exists>p \<in> Lset(i). p\<in>A & (\<exists>f \<in> Lset(i). \<exists>b \<in> Lset(i).
   256 	      \<exists>nb \<in> Lset(i). \<exists>cnbf \<in> Lset(i). 
   256               \<exists>nb \<in> Lset(i). \<exists>cnbf \<in> Lset(i).
   257 		pair(**Lset(i),f,b,p) & pair(**Lset(i),n,b,nb) & 
   257                 pair(**Lset(i),f,b,p) & pair(**Lset(i),n,b,nb) &
   258 		is_cons(**Lset(i),nb,f,cnbf) & upair(**Lset(i),cnbf,cnbf,z))]"
   258                 is_cons(**Lset(i),nb,f,cnbf) & upair(**Lset(i),cnbf,cnbf,z))]"
   259 by (intro FOL_reflections function_reflections)
   259 by (intro FOL_reflections function_reflections)
   260 
   260 
   261 lemma funspace_succ_replacement:
   261 lemma funspace_succ_replacement:
   262      "L(n) ==> 
   262      "L(n) ==>
   263       strong_replacement(L, \<lambda>p z. \<exists>f[L]. \<exists>b[L]. \<exists>nb[L]. \<exists>cnbf[L]. 
   263       strong_replacement(L, \<lambda>p z. \<exists>f[L]. \<exists>b[L]. \<exists>nb[L]. \<exists>cnbf[L].
   264                 pair(L,f,b,p) & pair(L,n,b,nb) & is_cons(L,nb,f,cnbf) &
   264                 pair(L,f,b,p) & pair(L,n,b,nb) & is_cons(L,nb,f,cnbf) &
   265                 upair(L,cnbf,cnbf,z))"
   265                 upair(L,cnbf,cnbf,z))"
   266 apply (rule strong_replacementI) 
   266 apply (rule strong_replacementI)
   267 apply (rule rallI) 
   267 apply (rule rallI)
   268 apply (rule separation_CollectI) 
   268 apply (rule separation_CollectI)
   269 apply (rule_tac A="{n,A,z}" in subset_LsetE, blast ) 
   269 apply (rule_tac A="{n,A,z}" in subset_LsetE, blast )
   270 apply (rule ReflectsE [OF funspace_succ_Reflects], assumption)
   270 apply (rule ReflectsE [OF funspace_succ_Reflects], assumption)
   271 apply (drule subset_Lset_ltD, assumption) 
   271 apply (drule subset_Lset_ltD, assumption)
   272 apply (erule reflection_imp_L_separation)
   272 apply (erule reflection_imp_L_separation)
   273   apply (simp_all add: lt_Ord2)
   273   apply (simp_all add: lt_Ord2)
   274 apply (rule DPow_LsetI)
   274 apply (rule DPow_LsetI)
   275 apply (rename_tac u) 
   275 apply (rename_tac u)
   276 apply (rule bex_iff_sats)
   276 apply (rule bex_iff_sats)
   277 apply (rule conj_iff_sats)
   277 apply (rule conj_iff_sats)
   278 apply (rule_tac env = "[p,u,n,A]" in mem_iff_sats) 
   278 apply (rule_tac env = "[p,u,n,A]" in mem_iff_sats)
   279 apply (rule sep_rules | simp)+
   279 apply (rule sep_rules | simp)+
   280 done
   280 done
   281 
   281 
   282 
   282 
   283 subsection{*Separation for Order-Isomorphisms*}
   283 subsection{*Separation for Order-Isomorphisms*}
   284 
   284 
   285 lemma well_ord_iso_Reflects:
   285 lemma well_ord_iso_Reflects:
   286   "REFLECTS[\<lambda>x. x\<in>A --> 
   286   "REFLECTS[\<lambda>x. x\<in>A -->
   287                 (\<exists>y[L]. \<exists>p[L]. fun_apply(L,f,x,y) & pair(L,y,x,p) & p \<in> r),
   287                 (\<exists>y[L]. \<exists>p[L]. fun_apply(L,f,x,y) & pair(L,y,x,p) & p \<in> r),
   288         \<lambda>i x. x\<in>A --> (\<exists>y \<in> Lset(i). \<exists>p \<in> Lset(i). 
   288         \<lambda>i x. x\<in>A --> (\<exists>y \<in> Lset(i). \<exists>p \<in> Lset(i).
   289                 fun_apply(**Lset(i),f,x,y) & pair(**Lset(i),y,x,p) & p \<in> r)]"
   289                 fun_apply(**Lset(i),f,x,y) & pair(**Lset(i),y,x,p) & p \<in> r)]"
   290 by (intro FOL_reflections function_reflections)
   290 by (intro FOL_reflections function_reflections)
   291 
   291 
   292 lemma well_ord_iso_separation:
   292 lemma well_ord_iso_separation:
   293      "[| L(A); L(f); L(r) |] 
   293      "[| L(A); L(f); L(r) |]
   294       ==> separation (L, \<lambda>x. x\<in>A --> (\<exists>y[L]. (\<exists>p[L]. 
   294       ==> separation (L, \<lambda>x. x\<in>A --> (\<exists>y[L]. (\<exists>p[L].
   295 		     fun_apply(L,f,x,y) & pair(L,y,x,p) & p \<in> r)))"
   295                      fun_apply(L,f,x,y) & pair(L,y,x,p) & p \<in> r)))"
   296 apply (rule separation_CollectI) 
   296 apply (rule separation_CollectI)
   297 apply (rule_tac A="{A,f,r,z}" in subset_LsetE, blast ) 
   297 apply (rule_tac A="{A,f,r,z}" in subset_LsetE, blast )
   298 apply (rule ReflectsE [OF well_ord_iso_Reflects], assumption)
   298 apply (rule ReflectsE [OF well_ord_iso_Reflects], assumption)
   299 apply (drule subset_Lset_ltD, assumption) 
   299 apply (drule subset_Lset_ltD, assumption)
   300 apply (erule reflection_imp_L_separation)
   300 apply (erule reflection_imp_L_separation)
   301   apply (simp_all add: lt_Ord2)
   301   apply (simp_all add: lt_Ord2)
   302 apply (rule DPow_LsetI)
   302 apply (rule DPow_LsetI)
   303 apply (rename_tac u) 
   303 apply (rename_tac u)
   304 apply (rule imp_iff_sats)
   304 apply (rule imp_iff_sats)
   305 apply (rule_tac env = "[u,A,f,r]" in mem_iff_sats) 
   305 apply (rule_tac env = "[u,A,f,r]" in mem_iff_sats)
   306 apply (rule sep_rules | simp)+
   306 apply (rule sep_rules | simp)+
   307 done
   307 done
   308 
   308 
   309 
   309 
   310 subsection{*Separation for @{term "obase"}*}
   310 subsection{*Separation for @{term "obase"}*}
   311 
   311 
   312 lemma obase_reflects:
   312 lemma obase_reflects:
   313   "REFLECTS[\<lambda>a. \<exists>x[L]. \<exists>g[L]. \<exists>mx[L]. \<exists>par[L]. 
   313   "REFLECTS[\<lambda>a. \<exists>x[L]. \<exists>g[L]. \<exists>mx[L]. \<exists>par[L].
   314 	     ordinal(L,x) & membership(L,x,mx) & pred_set(L,A,a,r,par) &
   314              ordinal(L,x) & membership(L,x,mx) & pred_set(L,A,a,r,par) &
   315 	     order_isomorphism(L,par,r,x,mx,g),
   315              order_isomorphism(L,par,r,x,mx,g),
   316         \<lambda>i a. \<exists>x \<in> Lset(i). \<exists>g \<in> Lset(i). \<exists>mx \<in> Lset(i). \<exists>par \<in> Lset(i). 
   316         \<lambda>i a. \<exists>x \<in> Lset(i). \<exists>g \<in> Lset(i). \<exists>mx \<in> Lset(i). \<exists>par \<in> Lset(i).
   317 	     ordinal(**Lset(i),x) & membership(**Lset(i),x,mx) & pred_set(**Lset(i),A,a,r,par) &
   317              ordinal(**Lset(i),x) & membership(**Lset(i),x,mx) & pred_set(**Lset(i),A,a,r,par) &
   318 	     order_isomorphism(**Lset(i),par,r,x,mx,g)]"
   318              order_isomorphism(**Lset(i),par,r,x,mx,g)]"
   319 by (intro FOL_reflections function_reflections fun_plus_reflections)
   319 by (intro FOL_reflections function_reflections fun_plus_reflections)
   320 
   320 
   321 lemma obase_separation:
   321 lemma obase_separation:
   322      --{*part of the order type formalization*}
   322      --{*part of the order type formalization*}
   323      "[| L(A); L(r) |] 
   323      "[| L(A); L(r) |]
   324       ==> separation(L, \<lambda>a. \<exists>x[L]. \<exists>g[L]. \<exists>mx[L]. \<exists>par[L]. 
   324       ==> separation(L, \<lambda>a. \<exists>x[L]. \<exists>g[L]. \<exists>mx[L]. \<exists>par[L].
   325 	     ordinal(L,x) & membership(L,x,mx) & pred_set(L,A,a,r,par) &
   325              ordinal(L,x) & membership(L,x,mx) & pred_set(L,A,a,r,par) &
   326 	     order_isomorphism(L,par,r,x,mx,g))"
   326              order_isomorphism(L,par,r,x,mx,g))"
   327 apply (rule separation_CollectI) 
   327 apply (rule separation_CollectI)
   328 apply (rule_tac A="{A,r,z}" in subset_LsetE, blast ) 
   328 apply (rule_tac A="{A,r,z}" in subset_LsetE, blast )
   329 apply (rule ReflectsE [OF obase_reflects], assumption)
   329 apply (rule ReflectsE [OF obase_reflects], assumption)
   330 apply (drule subset_Lset_ltD, assumption) 
   330 apply (drule subset_Lset_ltD, assumption)
   331 apply (erule reflection_imp_L_separation)
   331 apply (erule reflection_imp_L_separation)
   332   apply (simp_all add: lt_Ord2)
   332   apply (simp_all add: lt_Ord2)
   333 apply (rule DPow_LsetI)
   333 apply (rule DPow_LsetI)
   334 apply (rename_tac u) 
   334 apply (rename_tac u)
   335 apply (rule bex_iff_sats)
   335 apply (rule bex_iff_sats)
   336 apply (rule conj_iff_sats)
   336 apply (rule conj_iff_sats)
   337 apply (rule_tac env = "[x,u,A,r]" in ordinal_iff_sats) 
   337 apply (rule_tac env = "[x,u,A,r]" in ordinal_iff_sats)
   338 apply (rule sep_rules | simp)+
   338 apply (rule sep_rules | simp)+
   339 done
   339 done
   340 
   340 
   341 
   341 
   342 subsection{*Separation for a Theorem about @{term "obase"}*}
   342 subsection{*Separation for a Theorem about @{term "obase"}*}
   343 
   343 
   344 lemma obase_equals_reflects:
   344 lemma obase_equals_reflects:
   345   "REFLECTS[\<lambda>x. x\<in>A --> ~(\<exists>y[L]. \<exists>g[L]. 
   345   "REFLECTS[\<lambda>x. x\<in>A --> ~(\<exists>y[L]. \<exists>g[L].
   346 		ordinal(L,y) & (\<exists>my[L]. \<exists>pxr[L]. 
   346                 ordinal(L,y) & (\<exists>my[L]. \<exists>pxr[L].
   347 		membership(L,y,my) & pred_set(L,A,x,r,pxr) &
   347                 membership(L,y,my) & pred_set(L,A,x,r,pxr) &
   348 		order_isomorphism(L,pxr,r,y,my,g))),
   348                 order_isomorphism(L,pxr,r,y,my,g))),
   349 	\<lambda>i x. x\<in>A --> ~(\<exists>y \<in> Lset(i). \<exists>g \<in> Lset(i). 
   349         \<lambda>i x. x\<in>A --> ~(\<exists>y \<in> Lset(i). \<exists>g \<in> Lset(i).
   350 		ordinal(**Lset(i),y) & (\<exists>my \<in> Lset(i). \<exists>pxr \<in> Lset(i). 
   350                 ordinal(**Lset(i),y) & (\<exists>my \<in> Lset(i). \<exists>pxr \<in> Lset(i).
   351 		membership(**Lset(i),y,my) & pred_set(**Lset(i),A,x,r,pxr) &
   351                 membership(**Lset(i),y,my) & pred_set(**Lset(i),A,x,r,pxr) &
   352 		order_isomorphism(**Lset(i),pxr,r,y,my,g)))]"
   352                 order_isomorphism(**Lset(i),pxr,r,y,my,g)))]"
   353 by (intro FOL_reflections function_reflections fun_plus_reflections)
   353 by (intro FOL_reflections function_reflections fun_plus_reflections)
   354 
   354 
   355 
   355 
   356 lemma obase_equals_separation:
   356 lemma obase_equals_separation:
   357      "[| L(A); L(r) |] 
   357      "[| L(A); L(r) |]
   358       ==> separation (L, \<lambda>x. x\<in>A --> ~(\<exists>y[L]. \<exists>g[L]. 
   358       ==> separation (L, \<lambda>x. x\<in>A --> ~(\<exists>y[L]. \<exists>g[L].
   359 			      ordinal(L,y) & (\<exists>my[L]. \<exists>pxr[L]. 
   359                               ordinal(L,y) & (\<exists>my[L]. \<exists>pxr[L].
   360 			      membership(L,y,my) & pred_set(L,A,x,r,pxr) &
   360                               membership(L,y,my) & pred_set(L,A,x,r,pxr) &
   361 			      order_isomorphism(L,pxr,r,y,my,g))))"
   361                               order_isomorphism(L,pxr,r,y,my,g))))"
   362 apply (rule separation_CollectI) 
   362 apply (rule separation_CollectI)
   363 apply (rule_tac A="{A,r,z}" in subset_LsetE, blast ) 
   363 apply (rule_tac A="{A,r,z}" in subset_LsetE, blast )
   364 apply (rule ReflectsE [OF obase_equals_reflects], assumption)
   364 apply (rule ReflectsE [OF obase_equals_reflects], assumption)
   365 apply (drule subset_Lset_ltD, assumption) 
   365 apply (drule subset_Lset_ltD, assumption)
   366 apply (erule reflection_imp_L_separation)
   366 apply (erule reflection_imp_L_separation)
   367   apply (simp_all add: lt_Ord2)
   367   apply (simp_all add: lt_Ord2)
   368 apply (rule DPow_LsetI)
   368 apply (rule DPow_LsetI)
   369 apply (rename_tac u) 
   369 apply (rename_tac u)
   370 apply (rule imp_iff_sats ball_iff_sats disj_iff_sats not_iff_sats)+
   370 apply (rule imp_iff_sats ball_iff_sats disj_iff_sats not_iff_sats)+
   371 apply (rule_tac env = "[u,A,r]" in mem_iff_sats) 
   371 apply (rule_tac env = "[u,A,r]" in mem_iff_sats)
   372 apply (rule sep_rules | simp)+
   372 apply (rule sep_rules | simp)+
   373 done
   373 done
   374 
   374 
   375 
   375 
   376 subsection{*Replacement for @{term "omap"}*}
   376 subsection{*Replacement for @{term "omap"}*}
   377 
   377 
   378 lemma omap_reflects:
   378 lemma omap_reflects:
   379  "REFLECTS[\<lambda>z. \<exists>a[L]. a\<in>B & (\<exists>x[L]. \<exists>g[L]. \<exists>mx[L]. \<exists>par[L]. 
   379  "REFLECTS[\<lambda>z. \<exists>a[L]. a\<in>B & (\<exists>x[L]. \<exists>g[L]. \<exists>mx[L]. \<exists>par[L].
   380      ordinal(L,x) & pair(L,a,x,z) & membership(L,x,mx) & 
   380      ordinal(L,x) & pair(L,a,x,z) & membership(L,x,mx) &
   381      pred_set(L,A,a,r,par) & order_isomorphism(L,par,r,x,mx,g)),
   381      pred_set(L,A,a,r,par) & order_isomorphism(L,par,r,x,mx,g)),
   382  \<lambda>i z. \<exists>a \<in> Lset(i). a\<in>B & (\<exists>x \<in> Lset(i). \<exists>g \<in> Lset(i). \<exists>mx \<in> Lset(i). 
   382  \<lambda>i z. \<exists>a \<in> Lset(i). a\<in>B & (\<exists>x \<in> Lset(i). \<exists>g \<in> Lset(i). \<exists>mx \<in> Lset(i).
   383         \<exists>par \<in> Lset(i). 
   383         \<exists>par \<in> Lset(i).
   384 	 ordinal(**Lset(i),x) & pair(**Lset(i),a,x,z) & 
   384          ordinal(**Lset(i),x) & pair(**Lset(i),a,x,z) &
   385          membership(**Lset(i),x,mx) & pred_set(**Lset(i),A,a,r,par) & 
   385          membership(**Lset(i),x,mx) & pred_set(**Lset(i),A,a,r,par) &
   386          order_isomorphism(**Lset(i),par,r,x,mx,g))]"
   386          order_isomorphism(**Lset(i),par,r,x,mx,g))]"
   387 by (intro FOL_reflections function_reflections fun_plus_reflections)
   387 by (intro FOL_reflections function_reflections fun_plus_reflections)
   388 
   388 
   389 lemma omap_replacement:
   389 lemma omap_replacement:
   390      "[| L(A); L(r) |] 
   390      "[| L(A); L(r) |]
   391       ==> strong_replacement(L,
   391       ==> strong_replacement(L,
   392              \<lambda>a z. \<exists>x[L]. \<exists>g[L]. \<exists>mx[L]. \<exists>par[L]. 
   392              \<lambda>a z. \<exists>x[L]. \<exists>g[L]. \<exists>mx[L]. \<exists>par[L].
   393 	     ordinal(L,x) & pair(L,a,x,z) & membership(L,x,mx) & 
   393              ordinal(L,x) & pair(L,a,x,z) & membership(L,x,mx) &
   394 	     pred_set(L,A,a,r,par) & order_isomorphism(L,par,r,x,mx,g))"
   394              pred_set(L,A,a,r,par) & order_isomorphism(L,par,r,x,mx,g))"
   395 apply (rule strong_replacementI) 
   395 apply (rule strong_replacementI)
   396 apply (rule rallI)
   396 apply (rule rallI)
   397 apply (rename_tac B)  
   397 apply (rename_tac B)
   398 apply (rule separation_CollectI) 
   398 apply (rule separation_CollectI)
   399 apply (rule_tac A="{A,B,r,z}" in subset_LsetE, blast ) 
   399 apply (rule_tac A="{A,B,r,z}" in subset_LsetE, blast )
   400 apply (rule ReflectsE [OF omap_reflects], assumption)
   400 apply (rule ReflectsE [OF omap_reflects], assumption)
   401 apply (drule subset_Lset_ltD, assumption) 
   401 apply (drule subset_Lset_ltD, assumption)
   402 apply (erule reflection_imp_L_separation)
   402 apply (erule reflection_imp_L_separation)
   403   apply (simp_all add: lt_Ord2)
   403   apply (simp_all add: lt_Ord2)
   404 apply (rule DPow_LsetI)
   404 apply (rule DPow_LsetI)
   405 apply (rename_tac u) 
   405 apply (rename_tac u)
   406 apply (rule bex_iff_sats conj_iff_sats)+
   406 apply (rule bex_iff_sats conj_iff_sats)+
   407 apply (rule_tac env = "[a,u,A,B,r]" in mem_iff_sats) 
   407 apply (rule_tac env = "[a,u,A,B,r]" in mem_iff_sats)
   408 apply (rule sep_rules | simp)+
   408 apply (rule sep_rules | simp)+
   409 done
   409 done
   410 
   410 
   411 
   411 
   412 subsection{*Separation for a Theorem about @{term "obase"}*}
   412 subsection{*Separation for a Theorem about @{term "obase"}*}
   413 
   413 
   414 lemma is_recfun_reflects:
   414 lemma is_recfun_reflects:
   415   "REFLECTS[\<lambda>x. \<exists>xa[L]. \<exists>xb[L]. 
   415   "REFLECTS[\<lambda>x. \<exists>xa[L]. \<exists>xb[L].
   416                 pair(L,x,a,xa) & xa \<in> r & pair(L,x,b,xb) & xb \<in> r & 
   416                 pair(L,x,a,xa) & xa \<in> r & pair(L,x,b,xb) & xb \<in> r &
   417                 (\<exists>fx[L]. \<exists>gx[L]. fun_apply(L,f,x,fx) & fun_apply(L,g,x,gx) & 
   417                 (\<exists>fx[L]. \<exists>gx[L]. fun_apply(L,f,x,fx) & fun_apply(L,g,x,gx) &
   418                                    fx \<noteq> gx),
   418                                    fx \<noteq> gx),
   419    \<lambda>i x. \<exists>xa \<in> Lset(i). \<exists>xb \<in> Lset(i). 
   419    \<lambda>i x. \<exists>xa \<in> Lset(i). \<exists>xb \<in> Lset(i).
   420           pair(**Lset(i),x,a,xa) & xa \<in> r & pair(**Lset(i),x,b,xb) & xb \<in> r &
   420           pair(**Lset(i),x,a,xa) & xa \<in> r & pair(**Lset(i),x,b,xb) & xb \<in> r &
   421                 (\<exists>fx \<in> Lset(i). \<exists>gx \<in> Lset(i). fun_apply(**Lset(i),f,x,fx) & 
   421                 (\<exists>fx \<in> Lset(i). \<exists>gx \<in> Lset(i). fun_apply(**Lset(i),f,x,fx) &
   422                   fun_apply(**Lset(i),g,x,gx) & fx \<noteq> gx)]"
   422                   fun_apply(**Lset(i),g,x,gx) & fx \<noteq> gx)]"
   423 by (intro FOL_reflections function_reflections fun_plus_reflections)
   423 by (intro FOL_reflections function_reflections fun_plus_reflections)
   424 
   424 
   425 lemma is_recfun_separation:
   425 lemma is_recfun_separation:
   426      --{*for well-founded recursion*}
   426      --{*for well-founded recursion*}
   427      "[| L(r); L(f); L(g); L(a); L(b) |] 
   427      "[| L(r); L(f); L(g); L(a); L(b) |]
   428      ==> separation(L, 
   428      ==> separation(L,
   429             \<lambda>x. \<exists>xa[L]. \<exists>xb[L]. 
   429             \<lambda>x. \<exists>xa[L]. \<exists>xb[L].
   430                 pair(L,x,a,xa) & xa \<in> r & pair(L,x,b,xb) & xb \<in> r & 
   430                 pair(L,x,a,xa) & xa \<in> r & pair(L,x,b,xb) & xb \<in> r &
   431                 (\<exists>fx[L]. \<exists>gx[L]. fun_apply(L,f,x,fx) & fun_apply(L,g,x,gx) & 
   431                 (\<exists>fx[L]. \<exists>gx[L]. fun_apply(L,f,x,fx) & fun_apply(L,g,x,gx) &
   432                                    fx \<noteq> gx))"
   432                                    fx \<noteq> gx))"
   433 apply (rule separation_CollectI) 
   433 apply (rule separation_CollectI)
   434 apply (rule_tac A="{r,f,g,a,b,z}" in subset_LsetE, blast ) 
   434 apply (rule_tac A="{r,f,g,a,b,z}" in subset_LsetE, blast )
   435 apply (rule ReflectsE [OF is_recfun_reflects], assumption)
   435 apply (rule ReflectsE [OF is_recfun_reflects], assumption)
   436 apply (drule subset_Lset_ltD, assumption) 
   436 apply (drule subset_Lset_ltD, assumption)
   437 apply (erule reflection_imp_L_separation)
   437 apply (erule reflection_imp_L_separation)
   438   apply (simp_all add: lt_Ord2)
   438   apply (simp_all add: lt_Ord2)
   439 apply (rule DPow_LsetI)
   439 apply (rule DPow_LsetI)
   440 apply (rename_tac u) 
   440 apply (rename_tac u)
   441 apply (rule bex_iff_sats conj_iff_sats)+
   441 apply (rule bex_iff_sats conj_iff_sats)+
   442 apply (rule_tac env = "[xa,u,r,f,g,a,b]" in pair_iff_sats) 
   442 apply (rule_tac env = "[xa,u,r,f,g,a,b]" in pair_iff_sats)
   443 apply (rule sep_rules | simp)+
   443 apply (rule sep_rules | simp)+
   444 done
   444 done
   445 
   445 
   446 
   446 
   447 subsection{*Instantiating the locale @{text M_axioms}*}
   447 subsection{*Instantiating the locale @{text M_axioms}*}
   448 text{*Separation (and Strong Replacement) for basic set-theoretic constructions
   448 text{*Separation (and Strong Replacement) for basic set-theoretic constructions
   449 such as intersection, Cartesian Product and image.*}
   449 such as intersection, Cartesian Product and image.*}
   450 
   450 
   451 ML
   451 theorem M_axioms_axioms_L: "M_axioms_axioms(L)"
   452 {*
   452   apply (rule M_axioms_axioms.intro)
   453 val Inter_separation = thm "Inter_separation";
   453                apply (assumption | rule
   454 val cartprod_separation = thm "cartprod_separation";
   454                  Inter_separation cartprod_separation image_separation
   455 val image_separation = thm "image_separation";
   455                  converse_separation restrict_separation
   456 val converse_separation = thm "converse_separation";
   456                  comp_separation pred_separation Memrel_separation
   457 val restrict_separation = thm "restrict_separation";
   457                  funspace_succ_replacement well_ord_iso_separation
   458 val comp_separation = thm "comp_separation";
   458                  obase_separation obase_equals_separation
   459 val pred_separation = thm "pred_separation";
   459                  omap_replacement is_recfun_separation)+
   460 val Memrel_separation = thm "Memrel_separation";
   460   done
   461 val funspace_succ_replacement = thm "funspace_succ_replacement";
   461   
   462 val well_ord_iso_separation = thm "well_ord_iso_separation";
   462 theorem M_axioms_L: "PROP M_axioms(L)"
   463 val obase_separation = thm "obase_separation";
   463   apply (rule M_axioms.intro)
   464 val obase_equals_separation = thm "obase_equals_separation";
   464    apply (rule M_triv_axioms_L)
   465 val omap_replacement = thm "omap_replacement";
   465   apply (rule M_axioms_axioms_L)
   466 val is_recfun_separation = thm "is_recfun_separation";
   466   done
   467 
   467 
   468 val m_axioms = 
   468 lemmas cartprod_iff = M_axioms.cartprod_iff [OF M_axioms_L]
   469     [Inter_separation, cartprod_separation, image_separation, 
   469   and cartprod_closed = M_axioms.cartprod_closed [OF M_axioms_L]
   470      converse_separation, restrict_separation, comp_separation, 
   470   and sum_closed = M_axioms.sum_closed [OF M_axioms_L]
   471      pred_separation, Memrel_separation, funspace_succ_replacement, 
   471   and M_converse_iff = M_axioms.M_converse_iff [OF M_axioms_L]
   472      well_ord_iso_separation, obase_separation,
   472   and converse_closed = M_axioms.converse_closed [OF M_axioms_L]
   473      obase_equals_separation, omap_replacement, is_recfun_separation]
   473   and converse_abs = M_axioms.converse_abs [OF M_axioms_L]
   474 
   474   and image_closed = M_axioms.image_closed [OF M_axioms_L]
   475 fun axioms_L th =
   475   and vimage_abs = M_axioms.vimage_abs [OF M_axioms_L]
   476     kill_flex_triv_prems (m_axioms MRS (triv_axioms_L th));
   476   and vimage_closed = M_axioms.vimage_closed [OF M_axioms_L]
   477 
   477   and domain_abs = M_axioms.domain_abs [OF M_axioms_L]
   478 bind_thm ("cartprod_iff", axioms_L (thm "M_axioms.cartprod_iff"));
   478   and domain_closed = M_axioms.domain_closed [OF M_axioms_L]
   479 bind_thm ("cartprod_closed", axioms_L (thm "M_axioms.cartprod_closed"));
   479   and range_abs = M_axioms.range_abs [OF M_axioms_L]
   480 bind_thm ("sum_closed", axioms_L (thm "M_axioms.sum_closed"));
   480   and range_closed = M_axioms.range_closed [OF M_axioms_L]
   481 bind_thm ("M_converse_iff", axioms_L (thm "M_axioms.M_converse_iff"));
   481   and field_abs = M_axioms.field_abs [OF M_axioms_L]
   482 bind_thm ("converse_closed", axioms_L (thm "M_axioms.converse_closed"));
   482   and field_closed = M_axioms.field_closed [OF M_axioms_L]
   483 bind_thm ("converse_abs", axioms_L (thm "M_axioms.converse_abs"));
   483   and relation_abs = M_axioms.relation_abs [OF M_axioms_L]
   484 bind_thm ("image_closed", axioms_L (thm "M_axioms.image_closed"));
   484   and function_abs = M_axioms.function_abs [OF M_axioms_L]
   485 bind_thm ("vimage_abs", axioms_L (thm "M_axioms.vimage_abs"));
   485   and apply_closed = M_axioms.apply_closed [OF M_axioms_L]
   486 bind_thm ("vimage_closed", axioms_L (thm "M_axioms.vimage_closed"));
   486   and apply_abs = M_axioms.apply_abs [OF M_axioms_L]
   487 bind_thm ("domain_abs", axioms_L (thm "M_axioms.domain_abs"));
   487   and typed_function_abs = M_axioms.typed_function_abs [OF M_axioms_L]
   488 bind_thm ("domain_closed", axioms_L (thm "M_axioms.domain_closed"));
   488   and injection_abs = M_axioms.injection_abs [OF M_axioms_L]
   489 bind_thm ("range_abs", axioms_L (thm "M_axioms.range_abs"));
   489   and surjection_abs = M_axioms.surjection_abs [OF M_axioms_L]
   490 bind_thm ("range_closed", axioms_L (thm "M_axioms.range_closed"));
   490   and bijection_abs = M_axioms.bijection_abs [OF M_axioms_L]
   491 bind_thm ("field_abs", axioms_L (thm "M_axioms.field_abs"));
   491   and M_comp_iff = M_axioms.M_comp_iff [OF M_axioms_L]
   492 bind_thm ("field_closed", axioms_L (thm "M_axioms.field_closed"));
   492   and comp_closed = M_axioms.comp_closed [OF M_axioms_L]
   493 bind_thm ("relation_abs", axioms_L (thm "M_axioms.relation_abs"));
   493   and composition_abs = M_axioms.composition_abs [OF M_axioms_L]
   494 bind_thm ("function_abs", axioms_L (thm "M_axioms.function_abs"));
   494   and restriction_is_function = M_axioms.restriction_is_function [OF M_axioms_L]
   495 bind_thm ("apply_closed", axioms_L (thm "M_axioms.apply_closed"));
   495   and restriction_abs = M_axioms.restriction_abs [OF M_axioms_L]
   496 bind_thm ("apply_abs", axioms_L (thm "M_axioms.apply_abs"));
   496   and M_restrict_iff = M_axioms.M_restrict_iff [OF M_axioms_L]
   497 bind_thm ("typed_function_abs", axioms_L (thm "M_axioms.typed_function_abs"));
   497   and restrict_closed = M_axioms.restrict_closed [OF M_axioms_L]
   498 bind_thm ("injection_abs", axioms_L (thm "M_axioms.injection_abs"));
   498   and Inter_abs = M_axioms.Inter_abs [OF M_axioms_L]
   499 bind_thm ("surjection_abs", axioms_L (thm "M_axioms.surjection_abs"));
   499   and Inter_closed = M_axioms.Inter_closed [OF M_axioms_L]
   500 bind_thm ("bijection_abs", axioms_L (thm "M_axioms.bijection_abs"));
   500   and Int_closed = M_axioms.Int_closed [OF M_axioms_L]
   501 bind_thm ("M_comp_iff", axioms_L (thm "M_axioms.M_comp_iff"));
   501   and finite_fun_closed = M_axioms.finite_fun_closed [OF M_axioms_L]
   502 bind_thm ("comp_closed", axioms_L (thm "M_axioms.comp_closed"));
   502   and is_funspace_abs = M_axioms.is_funspace_abs [OF M_axioms_L]
   503 bind_thm ("composition_abs", axioms_L (thm "M_axioms.composition_abs"));
   503   and succ_fun_eq2 = M_axioms.succ_fun_eq2 [OF M_axioms_L]
   504 bind_thm ("restriction_is_function", axioms_L (thm "M_axioms.restriction_is_function"));
   504   and funspace_succ = M_axioms.funspace_succ [OF M_axioms_L]
   505 bind_thm ("restriction_abs", axioms_L (thm "M_axioms.restriction_abs"));
   505   and finite_funspace_closed = M_axioms.finite_funspace_closed [OF M_axioms_L]
   506 bind_thm ("M_restrict_iff", axioms_L (thm "M_axioms.M_restrict_iff"));
   506 
   507 bind_thm ("restrict_closed", axioms_L (thm "M_axioms.restrict_closed"));
   507 lemmas is_recfun_equal = M_axioms.is_recfun_equal [OF M_axioms_L]
   508 bind_thm ("Inter_abs", axioms_L (thm "M_axioms.Inter_abs"));
   508   and is_recfun_cut = M_axioms.is_recfun_cut [OF M_axioms_L]
   509 bind_thm ("Inter_closed", axioms_L (thm "M_axioms.Inter_closed"));
   509   and is_recfun_functional = M_axioms.is_recfun_functional [OF M_axioms_L]
   510 bind_thm ("Int_closed", axioms_L (thm "M_axioms.Int_closed"));
   510   and is_recfun_relativize = M_axioms.is_recfun_relativize [OF M_axioms_L]
   511 bind_thm ("finite_fun_closed", axioms_L (thm "M_axioms.finite_fun_closed"));
   511   and is_recfun_restrict = M_axioms.is_recfun_restrict [OF M_axioms_L]
   512 bind_thm ("is_funspace_abs", axioms_L (thm "M_axioms.is_funspace_abs"));
   512   and univalent_is_recfun = M_axioms.univalent_is_recfun [OF M_axioms_L]
   513 bind_thm ("succ_fun_eq2", axioms_L (thm "M_axioms.succ_fun_eq2"));
   513   and exists_is_recfun_indstep = M_axioms.exists_is_recfun_indstep [OF M_axioms_L]
   514 bind_thm ("funspace_succ", axioms_L (thm "M_axioms.funspace_succ"));
   514   and wellfounded_exists_is_recfun = M_axioms.wellfounded_exists_is_recfun [OF M_axioms_L]
   515 bind_thm ("finite_funspace_closed", axioms_L (thm "M_axioms.finite_funspace_closed"));
   515   and wf_exists_is_recfun = M_axioms.wf_exists_is_recfun [OF M_axioms_L]
   516 *}
   516   and is_recfun_abs = M_axioms.is_recfun_abs [OF M_axioms_L]
   517 
   517   and irreflexive_abs = M_axioms.irreflexive_abs [OF M_axioms_L]
   518 ML
   518   and transitive_rel_abs = M_axioms.transitive_rel_abs [OF M_axioms_L]
   519 {*
   519   and linear_rel_abs = M_axioms.linear_rel_abs [OF M_axioms_L]
   520 bind_thm ("is_recfun_equal", axioms_L (thm "M_axioms.is_recfun_equal"));  
   520   and wellordered_is_trans_on = M_axioms.wellordered_is_trans_on [OF M_axioms_L]
   521 bind_thm ("is_recfun_cut", axioms_L (thm "M_axioms.is_recfun_cut")); 
   521   and wellordered_is_linear = M_axioms.wellordered_is_linear [OF M_axioms_L]
   522 bind_thm ("is_recfun_functional", axioms_L (thm "M_axioms.is_recfun_functional"));
   522   and wellordered_is_wellfounded_on = M_axioms.wellordered_is_wellfounded_on [OF M_axioms_L]
   523 bind_thm ("is_recfun_relativize", axioms_L (thm "M_axioms.is_recfun_relativize"));
   523   and wellfounded_imp_wellfounded_on = M_axioms.wellfounded_imp_wellfounded_on [OF M_axioms_L]
   524 bind_thm ("is_recfun_restrict", axioms_L (thm "M_axioms.is_recfun_restrict"));
   524   and wellfounded_on_subset_A = M_axioms.wellfounded_on_subset_A [OF M_axioms_L]
   525 bind_thm ("univalent_is_recfun", axioms_L (thm "M_axioms.univalent_is_recfun"));
   525   and wellfounded_on_iff_wellfounded = M_axioms.wellfounded_on_iff_wellfounded [OF M_axioms_L]
   526 bind_thm ("exists_is_recfun_indstep", axioms_L (thm "M_axioms.exists_is_recfun_indstep"));
   526   and wellfounded_on_imp_wellfounded = M_axioms.wellfounded_on_imp_wellfounded [OF M_axioms_L]
   527 bind_thm ("wellfounded_exists_is_recfun", axioms_L (thm "M_axioms.wellfounded_exists_is_recfun"));
   527   and wellfounded_on_field_imp_wellfounded = M_axioms.wellfounded_on_field_imp_wellfounded [OF M_axioms_L]
   528 bind_thm ("wf_exists_is_recfun", axioms_L (thm "M_axioms.wf_exists_is_recfun")); 
   528   and wellfounded_iff_wellfounded_on_field = M_axioms.wellfounded_iff_wellfounded_on_field [OF M_axioms_L]
   529 bind_thm ("is_recfun_abs", axioms_L (thm "M_axioms.is_recfun_abs"));
   529   and wellfounded_induct = M_axioms.wellfounded_induct [OF M_axioms_L]
   530 bind_thm ("irreflexive_abs", axioms_L (thm "M_axioms.irreflexive_abs"));  
   530   and wellfounded_on_induct = M_axioms.wellfounded_on_induct [OF M_axioms_L]
   531 bind_thm ("transitive_rel_abs", axioms_L (thm "M_axioms.transitive_rel_abs"));  
   531   and wellfounded_on_induct2 = M_axioms.wellfounded_on_induct2 [OF M_axioms_L]
   532 bind_thm ("linear_rel_abs", axioms_L (thm "M_axioms.linear_rel_abs"));  
   532   and linear_imp_relativized = M_axioms.linear_imp_relativized [OF M_axioms_L]
   533 bind_thm ("wellordered_is_trans_on", axioms_L (thm "M_axioms.wellordered_is_trans_on")); 
   533   and trans_on_imp_relativized = M_axioms.trans_on_imp_relativized [OF M_axioms_L]
   534 bind_thm ("wellordered_is_linear", axioms_L (thm "M_axioms.wellordered_is_linear")); 
   534   and wf_on_imp_relativized = M_axioms.wf_on_imp_relativized [OF M_axioms_L]
   535 bind_thm ("wellordered_is_wellfounded_on", axioms_L (thm "M_axioms.wellordered_is_wellfounded_on")); 
   535   and wf_imp_relativized = M_axioms.wf_imp_relativized [OF M_axioms_L]
   536 bind_thm ("wellfounded_imp_wellfounded_on", axioms_L (thm "M_axioms.wellfounded_imp_wellfounded_on")); 
   536   and well_ord_imp_relativized = M_axioms.well_ord_imp_relativized [OF M_axioms_L]
   537 bind_thm ("wellfounded_on_subset_A", axioms_L (thm "M_axioms.wellfounded_on_subset_A"));
   537   and order_isomorphism_abs = M_axioms.order_isomorphism_abs [OF M_axioms_L]
   538 bind_thm ("wellfounded_on_iff_wellfounded", axioms_L (thm "M_axioms.wellfounded_on_iff_wellfounded"));
   538   and pred_set_abs = M_axioms.pred_set_abs [OF M_axioms_L]
   539 bind_thm ("wellfounded_on_imp_wellfounded", axioms_L (thm "M_axioms.wellfounded_on_imp_wellfounded"));
   539 
   540 bind_thm ("wellfounded_on_field_imp_wellfounded", axioms_L (thm "M_axioms.wellfounded_on_field_imp_wellfounded"));
   540 lemmas pred_closed = M_axioms.pred_closed [OF M_axioms_L]
   541 bind_thm ("wellfounded_iff_wellfounded_on_field", axioms_L (thm "M_axioms.wellfounded_iff_wellfounded_on_field"));
   541   and membership_abs = M_axioms.membership_abs [OF M_axioms_L]
   542 bind_thm ("wellfounded_induct", axioms_L (thm "M_axioms.wellfounded_induct")); 
   542   and M_Memrel_iff = M_axioms.M_Memrel_iff [OF M_axioms_L]
   543 bind_thm ("wellfounded_on_induct", axioms_L (thm "M_axioms.wellfounded_on_induct")); 
   543   and Memrel_closed = M_axioms.Memrel_closed [OF M_axioms_L]
   544 bind_thm ("wellfounded_on_induct2", axioms_L (thm "M_axioms.wellfounded_on_induct2")); 
   544   and wellordered_iso_predD = M_axioms.wellordered_iso_predD [OF M_axioms_L]
   545 bind_thm ("linear_imp_relativized", axioms_L (thm "M_axioms.linear_imp_relativized")); 
   545   and wellordered_iso_pred_eq = M_axioms.wellordered_iso_pred_eq [OF M_axioms_L]
   546 bind_thm ("trans_on_imp_relativized", axioms_L (thm "M_axioms.trans_on_imp_relativized")); 
   546   and wellfounded_on_asym = M_axioms.wellfounded_on_asym [OF M_axioms_L]
   547 bind_thm ("wf_on_imp_relativized", axioms_L (thm "M_axioms.wf_on_imp_relativized")); 
   547   and wellordered_asym = M_axioms.wellordered_asym [OF M_axioms_L]
   548 bind_thm ("wf_imp_relativized", axioms_L (thm "M_axioms.wf_imp_relativized")); 
   548   and ord_iso_pred_imp_lt = M_axioms.ord_iso_pred_imp_lt [OF M_axioms_L]
   549 bind_thm ("well_ord_imp_relativized", axioms_L (thm "M_axioms.well_ord_imp_relativized")); 
   549   and obase_iff = M_axioms.obase_iff [OF M_axioms_L]
   550 bind_thm ("order_isomorphism_abs", axioms_L (thm "M_axioms.order_isomorphism_abs"));  
   550   and omap_iff = M_axioms.omap_iff [OF M_axioms_L]
   551 bind_thm ("pred_set_abs", axioms_L (thm "M_axioms.pred_set_abs"));  
   551   and omap_unique = M_axioms.omap_unique [OF M_axioms_L]
   552 *}
   552   and omap_yields_Ord = M_axioms.omap_yields_Ord [OF M_axioms_L]
   553 
   553   and otype_iff = M_axioms.otype_iff [OF M_axioms_L]
   554 ML
   554   and otype_eq_range = M_axioms.otype_eq_range [OF M_axioms_L]
   555 {*
   555   and Ord_otype = M_axioms.Ord_otype [OF M_axioms_L]
   556 bind_thm ("pred_closed", axioms_L (thm "M_axioms.pred_closed"));  
   556   and domain_omap = M_axioms.domain_omap [OF M_axioms_L]
   557 bind_thm ("membership_abs", axioms_L (thm "M_axioms.membership_abs"));  
   557   and omap_subset = M_axioms.omap_subset [OF M_axioms_L]
   558 bind_thm ("M_Memrel_iff", axioms_L (thm "M_axioms.M_Memrel_iff"));
   558   and omap_funtype = M_axioms.omap_funtype [OF M_axioms_L]
   559 bind_thm ("Memrel_closed", axioms_L (thm "M_axioms.Memrel_closed"));  
   559   and wellordered_omap_bij = M_axioms.wellordered_omap_bij [OF M_axioms_L]
   560 bind_thm ("wellordered_iso_predD", axioms_L (thm "M_axioms.wellordered_iso_predD"));
   560   and omap_ord_iso = M_axioms.omap_ord_iso [OF M_axioms_L]
   561 bind_thm ("wellordered_iso_pred_eq", axioms_L (thm "M_axioms.wellordered_iso_pred_eq"));
   561   and Ord_omap_image_pred = M_axioms.Ord_omap_image_pred [OF M_axioms_L]
   562 bind_thm ("wellfounded_on_asym", axioms_L (thm "M_axioms.wellfounded_on_asym"));
   562   and restrict_omap_ord_iso = M_axioms.restrict_omap_ord_iso [OF M_axioms_L]
   563 bind_thm ("wellordered_asym", axioms_L (thm "M_axioms.wellordered_asym"));
   563   and obase_equals = M_axioms.obase_equals [OF M_axioms_L]
   564 bind_thm ("ord_iso_pred_imp_lt", axioms_L (thm "M_axioms.ord_iso_pred_imp_lt"));
   564   and omap_ord_iso_otype = M_axioms.omap_ord_iso_otype [OF M_axioms_L]
   565 bind_thm ("obase_iff", axioms_L (thm "M_axioms.obase_iff"));
   565   and obase_exists = M_axioms.obase_exists [OF M_axioms_L]
   566 bind_thm ("omap_iff", axioms_L (thm "M_axioms.omap_iff"));
   566   and omap_exists = M_axioms.omap_exists [OF M_axioms_L]
   567 bind_thm ("omap_unique", axioms_L (thm "M_axioms.omap_unique"));
   567   and otype_exists = M_axioms.otype_exists [OF M_axioms_L]
   568 bind_thm ("omap_yields_Ord", axioms_L (thm "M_axioms.omap_yields_Ord"));
   568   and omap_ord_iso_otype' = M_axioms.omap_ord_iso_otype' [OF M_axioms_L]
   569 bind_thm ("otype_iff", axioms_L (thm "M_axioms.otype_iff"));
   569   and ordertype_exists = M_axioms.ordertype_exists [OF M_axioms_L]
   570 bind_thm ("otype_eq_range", axioms_L (thm "M_axioms.otype_eq_range"));
   570   and relativized_imp_well_ord = M_axioms.relativized_imp_well_ord [OF M_axioms_L]
   571 bind_thm ("Ord_otype", axioms_L (thm "M_axioms.Ord_otype"));
   571   and well_ord_abs = M_axioms.well_ord_abs [OF M_axioms_L]
   572 bind_thm ("domain_omap", axioms_L (thm "M_axioms.domain_omap"));
   572 
   573 bind_thm ("omap_subset", axioms_L (thm "M_axioms.omap_subset")); 
       
   574 bind_thm ("omap_funtype", axioms_L (thm "M_axioms.omap_funtype")); 
       
   575 bind_thm ("wellordered_omap_bij", axioms_L (thm "M_axioms.wellordered_omap_bij"));
       
   576 bind_thm ("omap_ord_iso", axioms_L (thm "M_axioms.omap_ord_iso"));
       
   577 bind_thm ("Ord_omap_image_pred", axioms_L (thm "M_axioms.Ord_omap_image_pred"));
       
   578 bind_thm ("restrict_omap_ord_iso", axioms_L (thm "M_axioms.restrict_omap_ord_iso"));
       
   579 bind_thm ("obase_equals", axioms_L (thm "M_axioms.obase_equals")); 
       
   580 bind_thm ("omap_ord_iso_otype", axioms_L (thm "M_axioms.omap_ord_iso_otype"));
       
   581 bind_thm ("obase_exists", axioms_L (thm "M_axioms.obase_exists"));
       
   582 bind_thm ("omap_exists", axioms_L (thm "M_axioms.omap_exists"));
       
   583 bind_thm ("otype_exists", axioms_L (thm "M_axioms.otype_exists"));
       
   584 bind_thm ("omap_ord_iso_otype", axioms_L (thm "M_axioms.omap_ord_iso_otype"));
       
   585 bind_thm ("ordertype_exists", axioms_L (thm "M_axioms.ordertype_exists"));
       
   586 bind_thm ("relativized_imp_well_ord", axioms_L (thm "M_axioms.relativized_imp_well_ord")); 
       
   587 bind_thm ("well_ord_abs", axioms_L (thm "M_axioms.well_ord_abs"));  
       
   588 *}
       
   589 
   573 
   590 declare cartprod_closed [intro,simp]
   574 declare cartprod_closed [intro,simp]
   591 declare sum_closed [intro,simp]
   575 declare sum_closed [intro,simp]
   592 declare converse_closed [intro,simp]
   576 declare converse_closed [intro,simp]
   593 declare converse_abs [simp]
   577 declare converse_abs [simp]
   612 declare restriction_abs [simp]
   596 declare restriction_abs [simp]
   613 declare restrict_closed [intro,simp]
   597 declare restrict_closed [intro,simp]
   614 declare Inter_abs [simp]
   598 declare Inter_abs [simp]
   615 declare Inter_closed [intro,simp]
   599 declare Inter_closed [intro,simp]
   616 declare Int_closed [intro,simp]
   600 declare Int_closed [intro,simp]
   617 declare finite_fun_closed [rule_format]
       
   618 declare is_funspace_abs [simp]
   601 declare is_funspace_abs [simp]
   619 declare finite_funspace_closed [intro,simp]
   602 declare finite_funspace_closed [intro,simp]
   620 
   603 
   621 end
   604 end