src/HOL/Library/LaTeXsugar.thy
changeset 55114 0ee5c17f2207
parent 55077 4cf280104b85
parent 55111 5792f5106c40
child 55954 a29aefc88c8d
equal deleted inserted replaced
55102:761e40ce91bc 55114:0ee5c17f2207
   104       in Pretty.block [Thy_Output.pretty_term ctxt tc, Pretty.str " ::",
   104       in Pretty.block [Thy_Output.pretty_term ctxt tc, Pretty.str " ::",
   105             Pretty.brk 1, Syntax.pretty_typ ctxt (fastype_of tc)]
   105             Pretty.brk 1, Syntax.pretty_typ ctxt (fastype_of tc)]
   106       end
   106       end
   107   in
   107   in
   108     Thy_Output.antiquotation @{binding "const_typ"}
   108     Thy_Output.antiquotation @{binding "const_typ"}
   109      (Scan.lift Args.name_source)
   109      (Scan.lift Args.name_inner_syntax)
   110        (fn {source = src, context = ctxt, ...} => fn arg =>
   110        (fn {source = src, context = ctxt, ...} => fn arg =>
   111           Thy_Output.output ctxt
   111           Thy_Output.output ctxt
   112             (Thy_Output.maybe_pretty_source pretty ctxt src [arg]))
   112             (Thy_Output.maybe_pretty_source pretty ctxt src [arg]))
   113   end;
   113   end;
   114 *}
   114 *}