--- a/src/HOL/Subst/UTerm.thy Thu Dec 06 00:45:04 2001 +0100
+++ b/src/HOL/Subst/UTerm.thy Thu Dec 06 00:46:24 2001 +0100
@@ -7,7 +7,7 @@
Binary trees with leaves that are constants or variables.
*)
-UTerm = Finite + Datatype +
+UTerm = Main +
datatype 'a uterm = Var ('a)
| Const ('a)