src/ZF/Constructible/MetaExists.thy
changeset 58871 c399ae4b836f
parent 32960 69916a850301
child 60770 240563fbf41d
equal deleted inserted replaced
58870:e2c0d8ef29cb 58871:c399ae4b836f
     1 (*  Title:      ZF/Constructible/MetaExists.thy
     1 (*  Title:      ZF/Constructible/MetaExists.thy
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     3 *)
     3 *)
     4 
     4 
     5 header{*The meta-existential quantifier*}
     5 section{*The meta-existential quantifier*}
     6 
     6 
     7 theory MetaExists imports Main begin
     7 theory MetaExists imports Main begin
     8 
     8 
     9 text{*Allows quantification over any term having sort @{text logic}.  Used to
     9 text{*Allows quantification over any term having sort @{text logic}.  Used to
    10 quantify over classes.  Yields a proposition rather than a FOL formula.*}
    10 quantify over classes.  Yields a proposition rather than a FOL formula.*}