src/HOL/Library/Eval.thy
changeset 25502 9200b36280c0
parent 24994 c385c4eabb3b
child 25536 01753a944433
--- a/src/HOL/Library/Eval.thy	Thu Nov 29 07:55:46 2007 +0100
+++ b/src/HOL/Library/Eval.thy	Thu Nov 29 17:08:26 2007 +0100
@@ -35,16 +35,16 @@
 *}
 
 instance "prop" :: typ_of
-  "typ_of T \<equiv> STR ''prop'' {\<struct>} []" ..
+  "typ_of (T\<Colon>prop itself) \<equiv> STR ''prop'' {\<struct>} []" ..
 
 instance itself :: (typ_of) typ_of
-  "typ_of T \<equiv> STR ''itself'' {\<struct>} [typ_of TYPE('a\<Colon>typ_of)]" ..
+  "typ_of (T\<Colon>'a itself itself) \<equiv> STR ''itself'' {\<struct>} [typ_of TYPE('a\<Colon>typ_of)]" ..
 
 instance set :: (typ_of) typ_of
-  "typ_of T \<equiv> STR ''set'' {\<struct>} [typ_of TYPE('a\<Colon>typ_of)]" ..
+  "typ_of (T\<Colon>'a set itself) \<equiv> STR ''set'' {\<struct>} [typ_of TYPE('a\<Colon>typ_of)]" ..
 
 instance int :: typ_of
-  "typ_of T \<equiv> STR ''IntDef.int'' {\<struct>} []" ..
+  "typ_of (T\<Colon>int itself) \<equiv> STR ''IntDef.int'' {\<struct>} []" ..
 
 setup {*
 let