src/HOL/Real/Lubs.thy
author berghofe
Fri, 23 Oct 1998 22:36:15 +0200
changeset 5760 7e2cf2820684
parent 5078 7b5ea59c0275
child 7219 4e3f386c2e37
permissions -rw-r--r--
Added theorems True_not_False and False_not_True (for rep_datatype).

(*  Title       : Lubs.thy
    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