src/ZF/ZF.thy
changeset 3065 c57861f709d2
parent 2872 ac81a17f86f8
child 3068 b7562e452816
--- a/src/ZF/ZF.thy	Tue Apr 29 16:39:13 1997 +0200
+++ b/src/ZF/ZF.thy	Tue Apr 29 17:13:41 1997 +0200
@@ -149,6 +149,8 @@
   "@SUM"      :: [pttrn, i, i] => i        ("(3\\<Sigma> _\\<in>_./ _)" 10)
   "@Ball"     :: [pttrn, i, o] => o        ("(3\\<forall> _\\<in>_./ _)" 10)
   "@Bex"      :: [pttrn, i, o] => o        ("(3\\<exists> _\\<in>_./ _)" 10)
+  "@Tuple"    :: [i, is] => i              ("\\<langle>(_,/ _)\\<rangle>")
+  "@pttrn"    :: pttrns => pttrn           ("\\<langle>_\\<rangle>")
 
 
 defs