src/ZF/Constructible/Wellorderings.thy
changeset 13505 52a16cb7fefb
parent 13428 99e52e78eb65
child 13513 b9e14471629c
equal deleted inserted replaced
13504:59066e97b551 13505:52a16cb7fefb
       
     1 (*  Title:      ZF/Constructible/Wellorderings.thy
       
     2     ID:         $Id$
       
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
       
     4     Copyright   2002  University of Cambridge
       
     5 *)
       
     6 
     1 header {*Relativized Wellorderings*}
     7 header {*Relativized Wellorderings*}
     2 
     8 
     3 theory Wellorderings = Relative:
     9 theory Wellorderings = Relative:
     4 
    10 
     5 text{*We define functions analogous to @{term ordermap} @{term ordertype} 
    11 text{*We define functions analogous to @{term ordermap} @{term ordertype} 
    55      "M(A) ==> linear_rel(M,A,r) <-> linear(A,r)"
    61      "M(A) ==> linear_rel(M,A,r) <-> linear(A,r)"
    56 by (simp add: linear_rel_def linear_def)
    62 by (simp add: linear_rel_def linear_def)
    57 
    63 
    58 lemma (in M_axioms) wellordered_is_trans_on: 
    64 lemma (in M_axioms) wellordered_is_trans_on: 
    59     "[| wellordered(M,A,r); M(A) |] ==> trans[A](r)"
    65     "[| wellordered(M,A,r); M(A) |] ==> trans[A](r)"
    60 by (auto simp add: wellordered_def )
    66 by (auto simp add: wellordered_def)
    61 
    67 
    62 lemma (in M_axioms) wellordered_is_linear: 
    68 lemma (in M_axioms) wellordered_is_linear: 
    63     "[| wellordered(M,A,r); M(A) |] ==> linear(A,r)"
    69     "[| wellordered(M,A,r); M(A) |] ==> linear(A,r)"
    64 by (auto simp add: wellordered_def )
    70 by (auto simp add: wellordered_def)
    65 
    71 
    66 lemma (in M_axioms) wellordered_is_wellfounded_on: 
    72 lemma (in M_axioms) wellordered_is_wellfounded_on: 
    67     "[| wellordered(M,A,r); M(A) |] ==> wellfounded_on(M,A,r)"
    73     "[| wellordered(M,A,r); M(A) |] ==> wellfounded_on(M,A,r)"
    68 by (auto simp add: wellordered_def )
    74 by (auto simp add: wellordered_def)
    69 
    75 
    70 lemma (in M_axioms) wellfounded_imp_wellfounded_on: 
    76 lemma (in M_axioms) wellfounded_imp_wellfounded_on: 
    71     "[| wellfounded(M,r); M(A) |] ==> wellfounded_on(M,A,r)"
    77     "[| wellfounded(M,r); M(A) |] ==> wellfounded_on(M,A,r)"
    72 by (auto simp add: wellfounded_def wellfounded_on_def)
    78 by (auto simp add: wellfounded_def wellfounded_on_def)
    73 
    79 
   627 
   633 
   628 
   634 
   629 lemma (in M_axioms) relativized_imp_well_ord: 
   635 lemma (in M_axioms) relativized_imp_well_ord: 
   630      "[| wellordered(M,A,r); M(A); M(r) |] ==> well_ord(A,r)" 
   636      "[| wellordered(M,A,r); M(A); M(r) |] ==> well_ord(A,r)" 
   631 apply (insert ordertype_exists [of A r], simp)
   637 apply (insert ordertype_exists [of A r], simp)
   632 apply (blast intro: well_ord_ord_iso well_ord_Memrel )  
   638 apply (blast intro: well_ord_ord_iso well_ord_Memrel)  
   633 done
   639 done
   634 
   640 
   635 subsection {*Kunen's theorem 5.4, poage 127*}
   641 subsection {*Kunen's theorem 5.4, poage 127*}
   636 
   642 
   637 text{*(a) The notion of Wellordering is absolute*}
   643 text{*(a) The notion of Wellordering is absolute*}