equal
deleted
inserted
replaced
56 |
56 |
57 |
57 |
58 section \<open>Quick start\<close> |
58 section \<open>Quick start\<close> |
59 |
59 |
60 text \<open> |
60 text \<open> |
61 The starting point is a fresh installation of \<^bold>\<open>Ubuntu 20.04 or 22.04 |
61 The starting point is a fresh installation of \<^bold>\<open>Ubuntu 22.04 or 24.04 |
62 LTS\<close>\<^footnote>\<open>\<^url>\<open>https://ubuntu.com/download\<close>\<close>: these versions are mandatory due to |
62 LTS\<close>\<^footnote>\<open>\<^url>\<open>https://ubuntu.com/download\<close>\<close>: these versions are mandatory due to |
63 subtle dependencies on system packages and configuration that is assumed by |
63 subtle dependencies on system packages and configuration that is assumed by |
64 the Isabelle setup tool. |
64 the Isabelle setup tool. |
65 |
65 |
66 For production use, a proper \<^emph>\<open>Virtual Server\<close> or \<^emph>\<open>Root Server\<close> product |
66 For production use, a proper \<^emph>\<open>Virtual Server\<close> or \<^emph>\<open>Root Server\<close> product |
381 |
381 |
382 subsection \<open>\<^verbatim>\<open>isabelle phabricator_setup\<close>\<close> |
382 subsection \<open>\<^verbatim>\<open>isabelle phabricator_setup\<close>\<close> |
383 |
383 |
384 text \<open> |
384 text \<open> |
385 The @{tool_def phabricator_setup} tool installs a fresh Phorge instance |
385 The @{tool_def phabricator_setup} tool installs a fresh Phorge instance |
386 on Ubuntu 20.04 or 22.04 LTS: |
386 on Ubuntu 22.04 or 24.04 LTS: |
387 @{verbatim [display] \<open>Usage: isabelle phabricator_setup [OPTIONS] |
387 @{verbatim [display] \<open>Usage: isabelle phabricator_setup [OPTIONS] |
388 |
388 |
389 Options are: |
389 Options are: |
390 -M SOURCE install Mercurial from source: local PATH, or URL, or ":" |
390 -M SOURCE install Mercurial from source: local PATH, or URL, or ":" |
391 -R DIR repository directory (default: "/var/www/phabricator-NAME/repo") |
391 -R DIR repository directory (default: "/var/www/phabricator-NAME/repo") |
417 \<^medskip> |
417 \<^medskip> |
418 Option \<^verbatim>\<open>-U\<close> ensures a full update of system packages, before installing |
418 Option \<^verbatim>\<open>-U\<close> ensures a full update of system packages, before installing |
419 further packages required by Phorge. This might require a reboot. |
419 further packages required by Phorge. This might require a reboot. |
420 |
420 |
421 Option \<^verbatim>\<open>-M:\<close> installs a standard Mercurial release from source: a specific |
421 Option \<^verbatim>\<open>-M:\<close> installs a standard Mercurial release from source: a specific |
422 version that is known to work on Ubuntu 20.04 or 22.04, respectively. It is |
422 version that is known to work on Ubuntu 22.04 or 24.04, respectively. It is |
423 also possible to specify the path or URL of the source archive (\<^verbatim>\<open>.tar.gz\<close>). |
423 also possible to specify the path or URL of the source archive (\<^verbatim>\<open>.tar.gz\<close>). |
424 This option is recommended for production use, but it requires to |
424 This option is recommended for production use, but it requires to |
425 \<^emph>\<open>uninstall\<close> existing Mercurial packages provided by the operating system. |
425 \<^emph>\<open>uninstall\<close> existing Mercurial packages provided by the operating system. |
426 |
426 |
427 Option \<^verbatim>\<open>-n\<close> provides an alternative installation name. The default name |
427 Option \<^verbatim>\<open>-n\<close> provides an alternative installation name. The default name |