src/HOL/Real/Lubs.thy
author paulson
Mon, 16 Aug 1999 18:41:32 +0200
changeset 7219 4e3f386c2e37
parent 5078 7b5ea59c0275
child 7562 8519d5019309
permissions -rw-r--r--
inserted Id: lines

(*  Title       : Lubs.thy
    ID          : $Id$
    Author      : Jacques D. Fleuriot
    Copyright   : 1998  University of Cambridge
    Description : Upper bounds, lubs definitions
                  suggested by James Margetson
*) 


Lubs = Set +

consts
    
    "*<=" :: ['a set, 'a] => bool     (infixl 70)
    "<=*" :: ['a, 'a set] => bool     (infixl 70)

constdefs
    leastP      :: ['a =>bool,'a] => bool
    "leastP P x == (P x & x <=* Collect P)"

    isLub       :: ['a set, 'a set, 'a] => bool    
    "isLub R S x  == leastP (isUb R S) x"

    isUb        :: ['a set, 'a set, 'a] => bool     
    "isUb R S x   == S *<= x & x: R"

    ubs         :: ['a set, 'a set] => 'a set
    "ubs R S      == Collect (isUb R S)"

defs
    setle_def
    "S *<= x    == (ALL y: S. y <= x)"

    setge_def
    "x <=* S    == (ALL y: S. x <= y)"

end