src/ZF/Constructible/MetaExists.thy
changeset 21404 eb85850d3eb7
parent 21233 5a5c8ea5f66a
child 32960 69916a850301
equal deleted inserted replaced
21403:dd58f13a8eb4 21404:eb85850d3eb7
     9 
     9 
    10 text{*Allows quantification over any term having sort @{text logic}.  Used to
    10 text{*Allows quantification over any term having sort @{text logic}.  Used to
    11 quantify over classes.  Yields a proposition rather than a FOL formula.*}
    11 quantify over classes.  Yields a proposition rather than a FOL formula.*}
    12 
    12 
    13 definition
    13 definition
    14   ex :: "(('a::{}) => prop) => prop"            (binder "?? " 0)
    14   ex :: "(('a::{}) => prop) => prop"  (binder "?? " 0) where
    15   "ex(P) == (!!Q. (!!x. PROP P(x) ==> PROP Q) ==> PROP Q)"
    15   "ex(P) == (!!Q. (!!x. PROP P(x) ==> PROP Q) ==> PROP Q)"
    16 
    16 
    17 notation (xsymbols)
    17 notation (xsymbols)
    18   ex  (binder "\<Or>" 0)
    18   ex  (binder "\<Or>" 0)
    19 
    19