diff -r e5df9c8d9d4b -r bf085daea304 src/Doc/System/Server.thy --- a/src/Doc/System/Server.thy Mon Jun 08 15:09:57 2020 +0200 +++ b/src/Doc/System/Server.thy Mon Jun 08 21:38:41 2020 +0200 @@ -515,9 +515,9 @@ \<^item> \<^bold>\type\ \node = {node_name: string, theory_name: string}\ represents the internal node name of a theory. The \node_name\ is derived from the - canonical theory file-name (e.g.\ \<^verbatim>\"~~/src/HOL/ex/Seq.thy"\ after + canonical theory file-name (e.g.\ \<^verbatim>\"~~/src/HOL/Examples/Seq.thy"\ after normalization within the file-system). The \theory_name\ is the - session-qualified theory name (e.g.\ \<^verbatim>\HOL-ex.Seq\). + session-qualified theory name (e.g.\ \<^verbatim>\HOL-Examples.Seq\). \<^item> \<^bold>\type\ \node_status = {ok: bool, total: int, unprocessed: int, running: int, warned: int, failed: int, finished: int, canceled: bool, consolidated: @@ -975,8 +975,8 @@ The \master_dir\ field specifies the master directory of imported theories: it acts like the ``current working directory'' for locating theory files. This is irrelevant for \theories\ with an absolute path name (e.g.\ - \<^verbatim>\"~~/src/HOL/ex/Seq.thy"\) or session-qualified theory name (e.g.\ - \<^verbatim>\"HOL-ex/Seq"\). + \<^verbatim>\"~~/src/HOL/Examples/Seq.thy"\) or session-qualified theory name (e.g.\ + \<^verbatim>\"HOL-Examples.Seq"\). \<^medskip> The \pretty_margin\ field specifies the line width for pretty-printing. The @@ -1026,7 +1026,7 @@ Process some example theory from the Isabelle distribution, within the context of an already started session for Isabelle/HOL (see also \secref{sec:command-session-start}): - @{verbatim [display] \use_theories {"session_id": ..., "theories": ["~~/src/HOL/ex/Seq"]}\} + @{verbatim [display] \use_theories {"session_id": ..., "theories": ["~~/src/HOL/Examples/Seq"]}\} \<^medskip> Process some example theories in the context of their (single) parent