src/HOL/Typerep.thy
changeset 35430 df2862dc23a8
parent 35363 09489d8ffece
child 36176 3fe7e97ccca8
--- a/src/HOL/Typerep.thy	Wed Mar 03 00:28:22 2010 +0100
+++ b/src/HOL/Typerep.thy	Wed Mar 03 00:32:14 2010 +0100
@@ -33,7 +33,7 @@
 typed_print_translation {*
 let
   fun typerep_tr' show_sorts (*"typerep"*)
-          (Type (@{type_syntax fun}, [Type (@{type_syntax itself}, [T]), _]))
+          (Type (@{type_name fun}, [Type (@{type_name itself}, [T]), _]))
           (Const (@{const_syntax TYPE}, _) :: ts) =
         Term.list_comb
           (Syntax.const @{syntax_const "_TYPEREP"} $ Syntax.term_of_typ show_sorts T, ts)