diff -r 8891f4520d16 -r d8da44a8dd25 doc-src/Main/Docs/Main_Doc.thy --- a/doc-src/Main/Docs/Main_Doc.thy Fri Aug 27 00:09:56 2010 +0200 +++ b/doc-src/Main/Docs/Main_Doc.thy Fri Aug 27 12:40:20 2010 +0200 @@ -10,9 +10,9 @@ Syntax.pretty_typ ctxt T) val _ = Thy_Output.antiquotation "term_type_only" (Args.term -- Args.typ_abbrev) - (fn {source, context, ...} => fn arg => - Thy_Output.output - (Thy_Output.maybe_pretty_source (pretty_term_type_only context) source [arg])); + (fn {source, context = ctxt, ...} => fn arg => + Thy_Output.output ctxt + (Thy_Output.maybe_pretty_source pretty_term_type_only ctxt source [arg])); *} (*>*) text{*