src/Pure/Pure.thy
changeset 70009 435fb018e8ee
parent 69913 ca515cf61651
child 70047 96fe857a7a6f
--- a/src/Pure/Pure.thy	Thu Mar 28 21:22:44 2019 +0100
+++ b/src/Pure/Pure.thy	Thu Mar 28 21:24:55 2019 +0100
@@ -140,7 +140,7 @@
             val paths = Generated_Files.export_files thy other_thys;
           in
             if not (null paths) then
-              (writeln (Export.message thy "");
+              (writeln (Export.message thy Path.current);
                writeln (cat_lines (paths |> map (fn (path, pos) =>
                 Markup.markup (Markup.entityN, Position.def_properties_of pos)
                   (quote (Path.implode path))))))