src/ZF/ZF.thy
changeset 11322 6a20952757b2
parent 11233 34c81a796ee3
child 12114 a8e860c86252
--- a/src/ZF/ZF.thy	Mon May 21 14:52:27 2001 +0200
+++ b/src/ZF/ZF.thy	Mon May 21 14:53:11 2001 +0200
@@ -157,7 +157,7 @@
   "@UNION"    :: [pttrn, i, i] => i        ("(3\\<Union>_\\<in>_./ _)" 10)
   "@PROD"     :: [pttrn, i, i] => i        ("(3\\<Pi>_\\<in>_./ _)" 10)
   "@SUM"      :: [pttrn, i, i] => i        ("(3\\<Sigma>_\\<in>_./ _)" 10)
-  "@lam"      :: [pttrn, i, i] => i        ("(3\\<lambda>_:_./ _)" 10)
+  "@lam"      :: [pttrn, i, i] => i        ("(3\\<lambda>_\\<in>_./ _)" 10)
   "@Ball"     :: [pttrn, i, o] => o        ("(3\\<forall>_\\<in>_./ _)" 10)
   "@Bex"      :: [pttrn, i, o] => o        ("(3\\<exists>_\\<in>_./ _)" 10)