src/Pure/Pure.thy
changeset 73312 736b8853189a
parent 72841 fd8d82c4433b
child 73787 493b1ae188da
equal deleted inserted replaced
73311:54262af6d310 73312:736b8853189a
   134             val _ =
   134             val _ =
   135               (lines, pos0) |-> fold (fn line => fn pos1 =>
   135               (lines, pos0) |-> fold (fn line => fn pos1 =>
   136                 let
   136                 let
   137                   val pos2 = pos1 |> fold Position.advance (Symbol.explode line);
   137                   val pos2 = pos1 |> fold Position.advance (Symbol.explode line);
   138                   val range = Position.range (pos1, pos2);
   138                   val range = Position.range (pos1, pos2);
       
   139                   val source = Input.source true line range;
   139                   val _ =
   140                   val _ =
   140                     if line = "" then ()
   141                     if line = "" then ()
   141                     else if String.isPrefix "#" line then
   142                     else if String.isPrefix "#" line then
   142                       Context_Position.report ctxt (#1 range) Markup.comment
   143                       Context_Position.report ctxt (#1 range) Markup.comment
   143                     else
   144                     else
   144                       (ignore (Resources.check_dir ctxt (SOME dir) (Input.source true line range))
   145                       (ignore (Resources.check_session_dir ctxt (SOME dir) source)
   145                         handle ERROR msg => Output.error_message msg);
   146                         handle ERROR msg => Output.error_message msg);
   146                 in pos2 |> Position.advance "\n" end);
   147                 in pos2 |> Position.advance "\n" end);
   147           in thy' end)));
   148           in thy' end)));
   148 
   149 
   149   val _ =
   150   val _ =