src/Doc/System/Environment.thy
changeset 83319 6d1d2be24a24
parent 83007 b9715600883c
child 83320 7376008e7318
--- a/src/Doc/System/Environment.thy	Sun Oct 19 20:08:08 2025 +0200
+++ b/src/Doc/System/Environment.thy	Mon Oct 20 13:24:42 2025 +0200
@@ -8,8 +8,10 @@
 
 text \<open>
   This manual describes Isabelle together with related tools as seen from a
-  system oriented view. See also the \<^emph>\<open>Isabelle/Isar Reference Manual\<close> \<^cite>\<open>"isabelle-isar-ref"\<close> for the actual Isabelle input language and related
-  concepts, and \<^emph>\<open>The Isabelle/Isar Implementation Manual\<close> \<^cite>\<open>"isabelle-implementation"\<close> for the main concepts of the underlying
+  system oriented view. See also the \<^emph>\<open>Isabelle/Isar Reference Manual\<close>
+  \<^cite>\<open>"isabelle-isar-ref"\<close> for the actual Isabelle input language and
+  related concepts, and \<^emph>\<open>The Isabelle/Isar Implementation Manual\<close>
+  \<^cite>\<open>"isabelle-implementation"\<close> for the main concepts of the underlying
   implementation in Isabelle/ML.
 \<close>
 
@@ -101,10 +103,12 @@
   ISABELLE_HOME} yourself from the shell!
 
   \<^descr>[@{setting_def ISABELLE_HOME_USER}] is the user-specific counterpart of
-  @{setting ISABELLE_HOME}. The default value is relative to \<^path>\<open>$USER_HOME/.isabelle\<close>, under rare circumstances this may be changed in the
-  global setting file. Typically, the @{setting ISABELLE_HOME_USER} directory
-  mimics @{setting ISABELLE_HOME} to some extend. In particular, site-wide
-  defaults may be overridden by a private \<^verbatim>\<open>$ISABELLE_HOME_USER/etc/settings\<close>.
+  @{setting ISABELLE_HOME}. The default value is relative to
+  \<^path>\<open>$USER_HOME/.isabelle\<close>, under rare circumstances this may be changed
+  in the global setting file. Typically, the @{setting ISABELLE_HOME_USER}
+  directory mimics @{setting ISABELLE_HOME} to some extend. In particular,
+  site-wide defaults may be overridden by a private
+  \<^verbatim>\<open>$ISABELLE_HOME_USER/etc/settings\<close>.
 
   \<^descr>[@{setting_def ISABELLE_PLATFORM_FAMILY}\<open>\<^sup>*\<close>] is automatically set to the
   general platform family (\<^verbatim>\<open>linux\<close>, \<^verbatim>\<open>macos\<close>, \<^verbatim>\<open>windows\<close>). Note that