src/HOL/ex/CodeEval.thy
changeset 22473 753123c89d72
parent 22333 652f316ca26a
--- a/src/HOL/ex/CodeEval.thy	Mon Mar 19 19:28:27 2007 +0100
+++ b/src/HOL/ex/CodeEval.thy	Tue Mar 20 08:27:15 2007 +0100
@@ -10,7 +10,7 @@
 
 subsection {* The typ_of class *}
 
-class typ_of =
+class typ_of = type +
   fixes typ_of :: "'a itself \<Rightarrow> typ"
 
 ML {*