src/ZF/Constructible/MetaExists.thy
changeset 21233 5a5c8ea5f66a
parent 16417 9bc16273c2d4
child 21404 eb85850d3eb7
--- a/src/ZF/Constructible/MetaExists.thy	Tue Nov 07 19:39:54 2006 +0100
+++ b/src/ZF/Constructible/MetaExists.thy	Tue Nov 07 19:40:13 2006 +0100
@@ -10,12 +10,12 @@
 text{*Allows quantification over any term having sort @{text logic}.  Used to
 quantify over classes.  Yields a proposition rather than a FOL formula.*}
 
-constdefs
+definition
   ex :: "(('a::{}) => prop) => prop"            (binder "?? " 0)
   "ex(P) == (!!Q. (!!x. PROP P(x) ==> PROP Q) ==> PROP Q)"
 
-syntax (xsymbols)
-  "?? "        :: "[idts, o] => o"             ("(3\<Or>_./ _)" [0, 0] 0)
+notation (xsymbols)
+  ex  (binder "\<Or>" 0)
 
 lemma meta_exI: "PROP P(x) ==> (?? x. PROP P(x))"
 proof (unfold ex_def)