src/Doc/System/Phabricator.thy
changeset 81724 ed5a05b06ee0
parent 81717 114449035ec6
child 81731 3af5379aac0e
--- a/src/Doc/System/Phabricator.thy	Sat Jan 04 23:14:10 2025 +0100
+++ b/src/Doc/System/Phabricator.thy	Sat Jan 04 23:20:05 2025 +0100
@@ -58,7 +58,7 @@
 section \<open>Quick start\<close>
 
 text \<open>
-  The starting point is a fresh installation of \<^bold>\<open>Ubuntu 20.04 or 22.04
+  The starting point is a fresh installation of \<^bold>\<open>Ubuntu 22.04 or 24.04
   LTS\<close>\<^footnote>\<open>\<^url>\<open>https://ubuntu.com/download\<close>\<close>: these versions are mandatory due to
   subtle dependencies on system packages and configuration that is assumed by
   the Isabelle setup tool.
@@ -383,7 +383,7 @@
 
 text \<open>
   The @{tool_def phabricator_setup} tool installs a fresh Phorge instance
-  on Ubuntu 20.04 or 22.04 LTS:
+  on Ubuntu 22.04 or 24.04 LTS:
   @{verbatim [display] \<open>Usage: isabelle phabricator_setup [OPTIONS]
 
   Options are:
@@ -419,7 +419,7 @@
   further packages required by Phorge. This might require a reboot.
 
   Option \<^verbatim>\<open>-M:\<close> installs a standard Mercurial release from source: a specific
-  version that is known to work on Ubuntu 20.04 or 22.04, respectively. It is
+  version that is known to work on Ubuntu 22.04 or 24.04, respectively. It is
   also possible to specify the path or URL of the source archive (\<^verbatim>\<open>.tar.gz\<close>).
   This option is recommended for production use, but it requires to
   \<^emph>\<open>uninstall\<close> existing Mercurial packages provided by the operating system.