src/Doc/System/Environment.thy
changeset 83007 b9715600883c
parent 82984 98943be48607
child 83319 6d1d2be24a24
--- a/src/Doc/System/Environment.thy	Thu Aug 14 14:25:20 2025 +0100
+++ b/src/Doc/System/Environment.thy	Sat Aug 16 12:50:32 2025 +0200
@@ -305,10 +305,11 @@
 
 text \<open>
   The raw Isabelle ML process has limited use in actual applications: it lacks
-  the full session context that is required for Isabelle/ML/Scala integration
-  and Prover IDE messages or markup. It is better to use @{tool build}
-  (\secref{sec:tool-build}) for regular sessions, or its front-end @{tool
-  process_theories} (\secref{sec:tool-process-theories}) for adhoc sessions.
+  the full session context that is required for export artifacts,
+  Isabelle/ML/Scala integration and Prover IDE messages or markup. It is
+  better to use @{tool build} (\secref{sec:tool-build}) for regular sessions,
+  or its front-end @{tool process_theories}
+  (\secref{sec:tool-process-theories}) for adhoc sessions.
 \<close>