src/ZF/AC/first.thy
author paulson
Tue, 16 Jul 1996 15:49:46 +0200
changeset 1868 836950047d85
parent 1478 2b8c2a7547ab
permissions -rw-r--r--
Put in minimal simpset to avoid excessive simplification, just as in revision 1.9 of HOL/indrule.ML

(*  Title:      ZF/AC/first.thy
    ID:         $Id$
    Author:     Krzysztof Grabczewski

Theory helpful in proofs using first element of a well ordered set
*)

first = Order +

consts

  first                   :: [i, i, i] => o

defs

  first_def                "first(u, X, R) 
                            == u:X & (ALL v:X. v~=u --> <u,v> : R)"
end