src/HOL/Subst/UTLemmas.thy
changeset 1381 57777949b2f8
parent 968 3cdaa8724175
child 1476 608483c2122a
--- a/src/HOL/Subst/UTLemmas.thy	Fri Dec 01 12:27:09 1995 +0100
+++ b/src/HOL/Subst/UTLemmas.thy	Fri Dec 01 13:03:34 1995 +0100
@@ -9,8 +9,8 @@
 
 consts
 
-  vars_of       ::   "'a uterm=>'a set"
-  "<:"          ::   "['a uterm,'a uterm]=>bool"   (infixl 54) 
+  vars_of       ::   'a uterm=>'a set
+  "<:"          ::   ['a uterm,'a uterm]=>bool   (infixl 54) 
 
 rules  (*Definitions*)