src/ZF/ZF.thy
changeset 3065 c57861f709d2
parent 2872 ac81a17f86f8
child 3068 b7562e452816
equal deleted inserted replaced
3064:f04f93e5c0a9 3065:c57861f709d2
   147   "@UNION"    :: [pttrn, i, i] => i        ("(3\\<Union> _\\<in>_./ _)" 10)
   147   "@UNION"    :: [pttrn, i, i] => i        ("(3\\<Union> _\\<in>_./ _)" 10)
   148   "@PROD"     :: [pttrn, i, i] => i        ("(3\\<Pi> _\\<in>_./ _)" 10)
   148   "@PROD"     :: [pttrn, i, i] => i        ("(3\\<Pi> _\\<in>_./ _)" 10)
   149   "@SUM"      :: [pttrn, i, i] => i        ("(3\\<Sigma> _\\<in>_./ _)" 10)
   149   "@SUM"      :: [pttrn, i, i] => i        ("(3\\<Sigma> _\\<in>_./ _)" 10)
   150   "@Ball"     :: [pttrn, i, o] => o        ("(3\\<forall> _\\<in>_./ _)" 10)
   150   "@Ball"     :: [pttrn, i, o] => o        ("(3\\<forall> _\\<in>_./ _)" 10)
   151   "@Bex"      :: [pttrn, i, o] => o        ("(3\\<exists> _\\<in>_./ _)" 10)
   151   "@Bex"      :: [pttrn, i, o] => o        ("(3\\<exists> _\\<in>_./ _)" 10)
       
   152   "@Tuple"    :: [i, is] => i              ("\\<langle>(_,/ _)\\<rangle>")
       
   153   "@pttrn"    :: pttrns => pttrn           ("\\<langle>_\\<rangle>")
   152 
   154 
   153 
   155 
   154 defs
   156 defs
   155 
   157 
   156   (* Bounded Quantifiers *)
   158   (* Bounded Quantifiers *)