doc-src/Intro/list.thy
author chaieb
Wed, 19 May 2004 11:23:59 +0200
changeset 14758 af3b71a46a1c
parent 105 216d6ed87399
child 32960 69916a850301
permissions -rw-r--r--
A new implementation for presburger arithmetic following the one suggested in technical report Chaieb Amine and Tobias Nipkow. It is generic an smaller. the tactic has also changed and allows the abstaction over fuction occurences whose type is nat or int.
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