Subst/UTerm.thy
changeset 48 21291189b51e
parent 0 7949f97df77a
child 126 872f866e630f
--- a/Subst/UTerm.thy	Thu Feb 24 14:45:57 1994 +0100
+++ b/Subst/UTerm.thy	Wed Mar 02 12:26:55 1994 +0100
@@ -37,7 +37,7 @@
      (*defining the concrete constructors*)
   VAR_def  	"VAR(v) == In0(v)"
   CONST_def  	"CONST(v) == In1(In0(v))"
-  COMB_def 	"COMB(t,u) == In1(In1(t . u))"
+  COMB_def 	"COMB(t,u) == In1(In1(t $ u))"
      (*defining the abstract constructors*)
   Var_def  	"Var(v) == Abs_UTerm(VAR(Leaf(v)))"
   Const_def  	"Const(c) == Abs_UTerm(CONST(Leaf(c)))"