src/HOL/Typerep.thy
changeset 42247 12fe41a92cd5
parent 42245 29e3967550d5
child 43329 84472e198515
--- a/src/HOL/Typerep.thy	Wed Apr 06 13:27:59 2011 +0200
+++ b/src/HOL/Typerep.thy	Wed Apr 06 13:33:46 2011 +0200
@@ -30,13 +30,13 @@
 in [(@{syntax_const "_TYPEREP"}, typerep_tr)] end
 *}
 
-typed_print_translation {*
+typed_print_translation (advanced) {*
 let
-  fun typerep_tr' show_sorts (*"typerep"*)
+  fun typerep_tr' ctxt (*"typerep"*)
           (Type (@{type_name fun}, [Type (@{type_name itself}, [T]), _]))
           (Const (@{const_syntax TYPE}, _) :: ts) =
         Term.list_comb
-          (Syntax.const @{syntax_const "_TYPEREP"} $ Syntax_Phases.term_of_typ show_sorts T, ts)
+          (Syntax.const @{syntax_const "_TYPEREP"} $ Syntax_Phases.term_of_typ ctxt T, ts)
     | typerep_tr' _ T ts = raise Match;
 in [(@{const_syntax typerep}, typerep_tr')] end
 *}