src/ZF/AC/first.thy
changeset 1478 2b8c2a7547ab
parent 1401 0c439768f45c
equal deleted inserted replaced
1477:4c51ab632cda 1478:2b8c2a7547ab
     1 (*  Title: 	ZF/AC/first.thy
     1 (*  Title:      ZF/AC/first.thy
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author: 	Krzysztof Grabczewski
     3     Author:     Krzysztof Grabczewski
     4 
     4 
     5 Theory helpful in proofs using first element of a well ordered set
     5 Theory helpful in proofs using first element of a well ordered set
     6 *)
     6 *)
     7 
     7 
     8 first = Order +
     8 first = Order +
    12   first                   :: [i, i, i] => o
    12   first                   :: [i, i, i] => o
    13 
    13 
    14 defs
    14 defs
    15 
    15 
    16   first_def                "first(u, X, R) 
    16   first_def                "first(u, X, R) 
    17 			    == u:X & (ALL v:X. v~=u --> <u,v> : R)"
    17                             == u:X & (ALL v:X. v~=u --> <u,v> : R)"
    18 end
    18 end