doc-src/Intro/list.thy
author kleing
Wed, 11 Feb 2009 16:03:10 +1100
changeset 29858 c8cee17d7e50
parent 105 216d6ed87399
child 32960 69916a850301
permissions -rw-r--r--
Autosolve feature for detecting duplicate theorems; patch by Timothy Bourke
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
105
216d6ed87399 Initial revision
lcp
parents:
diff changeset
     1
List = FOL +
216d6ed87399 Initial revision
lcp
parents:
diff changeset
     2
types 	list 1
216d6ed87399 Initial revision
lcp
parents:
diff changeset
     3
arities list	:: (term)term
216d6ed87399 Initial revision
lcp
parents:
diff changeset
     4
consts	Nil	:: "'a list"
216d6ed87399 Initial revision
lcp
parents:
diff changeset
     5
   	Cons	:: "['a, 'a list] => 'a list" 
216d6ed87399 Initial revision
lcp
parents:
diff changeset
     6
end