src/CCL/Set.thy
changeset 42156 df219e736a5d
parent 41526 54b4686704af
child 48475 02dd825f5a4e
equal deleted inserted replaced
42155:ffe99b07c9c0 42156:df219e736a5d
    44   "INT x:A. B"  == "CONST INTER(A, %x. B)"
    44   "INT x:A. B"  == "CONST INTER(A, %x. B)"
    45   "UN x:A. B"   == "CONST UNION(A, %x. B)"
    45   "UN x:A. B"   == "CONST UNION(A, %x. B)"
    46   "ALL x:A. P"  == "CONST Ball(A, %x. P)"
    46   "ALL x:A. P"  == "CONST Ball(A, %x. P)"
    47   "EX x:A. P"   == "CONST Bex(A, %x. P)"
    47   "EX x:A. P"   == "CONST Bex(A, %x. P)"
    48 
    48 
    49 axioms
    49 axiomatization where
    50   mem_Collect_iff:       "(a : {x. P(x)}) <-> P(a)"
    50   mem_Collect_iff: "(a : {x. P(x)}) <-> P(a)" and
    51   set_extension:         "A=B <-> (ALL x. x:A <-> x:B)"
    51   set_extension: "A = B <-> (ALL x. x:A <-> x:B)"
    52 
    52 
    53 defs
    53 defs
    54   Ball_def:      "Ball(A, P)  == ALL x. x:A --> P(x)"
    54   Ball_def:      "Ball(A, P)  == ALL x. x:A --> P(x)"
    55   Bex_def:       "Bex(A, P)   == EX x. x:A & P(x)"
    55   Bex_def:       "Bex(A, P)   == EX x. x:A & P(x)"
    56   mono_def:      "mono(f)     == (ALL A B. A <= B --> f(A) <= f(B))"
    56   mono_def:      "mono(f)     == (ALL A B. A <= B --> f(A) <= f(B))"