src/ZF/List.thy
changeset 581 465075fd257b
parent 516 1957113f0d7d
child 753 ec86863e87c8
--- a/src/ZF/List.thy	Wed Aug 31 17:34:12 1994 +0200
+++ b/src/ZF/List.thy	Tue Sep 06 11:02:16 1994 +0200
@@ -30,7 +30,7 @@
 
   
 datatype
-  "list(A)" = "Nil" | "Cons" ("a:A", "l: list(A)")
+  "list(A)" = Nil | Cons ("a:A", "l: list(A)")
 
 
 translations