src/FOLP/ex/Prolog.thy
changeset 353 b5030aaca2ab
parent 0 a5a9c433f639
child 1466 bf18d174e9f8
--- a/src/FOLP/ex/Prolog.thy	Tue May 03 15:00:00 1994 +0200
+++ b/src/FOLP/ex/Prolog.thy	Tue May 03 15:14:54 1994 +0200
@@ -9,7 +9,7 @@
 *)
 
 Prolog = FOL +
-types   list 1
+types   'a list
 arities list    :: (term)term
 consts  Nil     :: "'a list"
         ":"     :: "['a, 'a list]=> 'a list"            (infixr 60)