src/Pure/PIDE/resources.ML
changeset 74789 a5c23da73fca
parent 74696 0554a5c4c191
child 74790 3ce6fb9db485
equal deleted inserted replaced
74788:95e514137861 74789:a5c23da73fca
   416 
   416 
   417 fun document_antiq (check: Proof.context -> Path.T option -> Input.source -> Path.T) =
   417 fun document_antiq (check: Proof.context -> Path.T option -> Input.source -> Path.T) =
   418   Args.context -- Scan.lift Parse.path_input >> (fn (ctxt, source) =>
   418   Args.context -- Scan.lift Parse.path_input >> (fn (ctxt, source) =>
   419    (check ctxt NONE source;
   419    (check ctxt NONE source;
   420     Latex.string (Latex.output_ascii_breakable "/" (Input.string_of source))
   420     Latex.string (Latex.output_ascii_breakable "/" (Input.string_of source))
   421     |> Latex.enclose_text "\\isatt{" "}"));
   421     |> XML.enclose "\\isatt{" "}"));
   422 
   422 
   423 fun ML_antiq check =
   423 fun ML_antiq check =
   424   Args.context -- Scan.lift Parse.path_input >> (fn (ctxt, source) =>
   424   Args.context -- Scan.lift Parse.path_input >> (fn (ctxt, source) =>
   425     check ctxt (SOME Path.current) source |> ML_Syntax.print_path);
   425     check ctxt (SOME Path.current) source |> ML_Syntax.print_path);
   426 
   426