src/ZF/ZF.thy
changeset 3068 b7562e452816
parent 3065 c57861f709d2
child 3692 9f9bcce140ce
--- a/src/ZF/ZF.thy	Tue Apr 29 17:23:53 1997 +0200
+++ b/src/ZF/ZF.thy	Tue Apr 29 17:38:02 1997 +0200
@@ -149,8 +149,10 @@
   "@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