src/Pure/Pure.thy
changeset 73312 736b8853189a
parent 72841 fd8d82c4433b
child 73787 493b1ae188da
--- a/src/Pure/Pure.thy	Sat Feb 27 13:37:04 2021 +0100
+++ b/src/Pure/Pure.thy	Sat Feb 27 13:39:06 2021 +0100
@@ -136,12 +136,13 @@
                 let
                   val pos2 = pos1 |> fold Position.advance (Symbol.explode line);
                   val range = Position.range (pos1, pos2);
+                  val source = Input.source true line range;
                   val _ =
                     if line = "" then ()
                     else if String.isPrefix "#" line then
                       Context_Position.report ctxt (#1 range) Markup.comment
                     else
-                      (ignore (Resources.check_dir ctxt (SOME dir) (Input.source true line range))
+                      (ignore (Resources.check_session_dir ctxt (SOME dir) source)
                         handle ERROR msg => Output.error_message msg);
                 in pos2 |> Position.advance "\n" end);
           in thy' end)));