- Datatype package now also supports arbitrarily branching datatypes
(using function types).
- Added new simplification procedure for proving distinctness of
constructors.
- dtK is now a reference.
Itrev = Main +
consts itrev :: 'a list => 'a list => 'a list
primrec
"itrev [] ys = ys"
"itrev (x#xs) ys = itrev xs (x#ys)"
end