src/HOL/Subst/UTerm.thy
changeset 12406 c9775847ed66
parent 5184 9b8547a9496a
child 15635 8408a06590a6
--- 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)