doc-src/Intro/list.thy
author wenzelm
Tue, 05 Jul 2011 22:38:44 +0200
changeset 43672 e9f26e66692d
parent 32960 69916a850301
permissions -rw-r--r--
theory name needs to conform to Path syntax;

List = FOL +
types   list 1
arities list    :: (term)term
consts  Nil     :: "'a list"
        Cons    :: "['a, 'a list] => 'a list" 
end