doc-src/Intro/list.thy
changeset 48941 fbf60999dc31
parent 48940 f0d87c6b7a2e
child 48942 75d8778f94d3
--- a/doc-src/Intro/list.thy	Mon Aug 27 20:19:09 2012 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,6 +0,0 @@
-List = FOL +
-types   list 1
-arities list    :: (term)term
-consts  Nil     :: "'a list"
-        Cons    :: "['a, 'a list] => 'a list" 
-end