src/HOL/HOL.thy
changeset 21410 c212b002fc8c
parent 21404 eb85850d3eb7
child 21486 b1fdc0513812
equal deleted inserted replaced
21409:6aa28caa96c5 21410:c212b002fc8c
   206 translations
   206 translations
   207   (index) "\<^sub>1" => (index) "\<^bsub>\<struct>\<^esub>"
   207   (index) "\<^sub>1" => (index) "\<^bsub>\<struct>\<^esub>"
   208 
   208 
   209 typed_print_translation {*
   209 typed_print_translation {*
   210 let
   210 let
   211   val syntax_name = Sign.const_syntax_name (the_context ());
   211   val thy = the_context ();
   212   fun tr' c = (c, fn show_sorts => fn T => fn ts =>
   212   fun tr' c = (c, fn show_sorts => fn T => fn ts =>
   213     if T = dummyT orelse not (! show_types) andalso can Term.dest_Type T then raise Match
   213     if T = dummyT orelse not (! show_types) andalso can Term.dest_Type T then raise Match
   214     else Syntax.const Syntax.constrainC $ Syntax.const c $ Syntax.term_of_typ show_sorts T);
   214     else Syntax.const Syntax.constrainC $ Syntax.const c $ Syntax.term_of_typ show_sorts T);
   215 in map (tr' o Sign.const_syntax_name (the_context ())) ["HOL.one", "HOL.zero"] end;
   215 in map (tr' o Sign.const_syntax_name thy) ["HOL.one", "HOL.zero"] end;
   216 *} -- {* show types that are presumably too general *}
   216 *} -- {* show types that are presumably too general *}
   217 
   217 
   218 notation
   218 notation
   219   uminus  ("- _" [81] 80)
   219   uminus  ("- _" [81] 80)
   220 
   220