src/Doc/System/Phabricator.thy
changeset 73534 e7fb17bca374
parent 72521 354bfab78cbf
child 75161 95612f330c93
equal deleted inserted replaced
73533:543d5539306d 73534:e7fb17bca374
    61 
    61 
    62 
    62 
    63 section \<open>Quick start\<close>
    63 section \<open>Quick start\<close>
    64 
    64 
    65 text \<open>
    65 text \<open>
    66   The starting point is a fresh installation of \<^bold>\<open>Ubuntu 18.04 or 20.04
    66   The starting point is a fresh installation of \<^bold>\<open>Ubuntu 20.04
    67   LTS\<close>\<^footnote>\<open>\<^url>\<open>https://ubuntu.com/download\<close>\<close>: this version is mandatory due to
    67   LTS\<close>\<^footnote>\<open>\<^url>\<open>https://ubuntu.com/download\<close>\<close>: this version is mandatory due to
    68   subtle dependencies on system packages and configuration that is assumed by
    68   subtle dependencies on system packages and configuration that is assumed by
    69   the Isabelle setup tool.
    69   the Isabelle setup tool.
    70 
    70 
    71   For production use, a proper \<^emph>\<open>Virtual Server\<close> or \<^emph>\<open>Root Server\<close> product
    71   For production use, a proper \<^emph>\<open>Virtual Server\<close> or \<^emph>\<open>Root Server\<close> product
   231 
   231 
   232     Then reload (or restart) Apache like this:
   232     Then reload (or restart) Apache like this:
   233     @{verbatim [display] \<open>  systemctl reload apache2\<close>}
   233     @{verbatim [display] \<open>  systemctl reload apache2\<close>}
   234 
   234 
   235     \<^item> Install \<^verbatim>\<open>certbot\<close> from \<^url>\<open>https://certbot.eff.org\<close> following the
   235     \<^item> Install \<^verbatim>\<open>certbot\<close> from \<^url>\<open>https://certbot.eff.org\<close> following the
   236     description for Apache and Ubuntu 18.04 or 20.04 on
   236     description for Apache and Ubuntu 20.04 on
   237     \<^url>\<open>https://certbot.eff.org/lets-encrypt/ubuntubionic-apache\<close>. Run
   237     \<^url>\<open>https://certbot.eff.org/lets-encrypt/ubuntubionic-apache\<close>. Run
   238     \<^verbatim>\<open>certbot\<close> interactively and let it operate on the domain
   238     \<^verbatim>\<open>certbot\<close> interactively and let it operate on the domain
   239     \<^verbatim>\<open>vcs.example.org\<close>.
   239     \<^verbatim>\<open>vcs.example.org\<close>.
   240 
   240 
   241     \<^item> Inform Phabricator about its new domain name like this:
   241     \<^item> Inform Phabricator about its new domain name like this:
   388 
   388 
   389 subsection \<open>\<^verbatim>\<open>isabelle phabricator_setup\<close>\<close>
   389 subsection \<open>\<^verbatim>\<open>isabelle phabricator_setup\<close>\<close>
   390 
   390 
   391 text \<open>
   391 text \<open>
   392   The @{tool_def phabricator_setup} tool installs a fresh Phabricator instance
   392   The @{tool_def phabricator_setup} tool installs a fresh Phabricator instance
   393   on Ubuntu 18.04 or 20.04 LTS:
   393   on Ubuntu 20.04 LTS:
   394   @{verbatim [display] \<open>Usage: isabelle phabricator_setup [OPTIONS]
   394   @{verbatim [display] \<open>Usage: isabelle phabricator_setup [OPTIONS]
   395 
   395 
   396   Options are:
   396   Options are:
   397     -M SOURCE    install Mercurial from source: local PATH, or URL, or ":"
   397     -M SOURCE    install Mercurial from source: local PATH, or URL, or ":"
   398     -R DIR       repository directory (default: "/var/www/phabricator-NAME/repo")
   398     -R DIR       repository directory (default: "/var/www/phabricator-NAME/repo")
   426   further packages required by Phabricator. This might require a reboot.
   426   further packages required by Phabricator. This might require a reboot.
   427 
   427 
   428   Option \<^verbatim>\<open>-M:\<close> installs a standard Mercurial release from source --- the one
   428   Option \<^verbatim>\<open>-M:\<close> installs a standard Mercurial release from source --- the one
   429   that is used by the Phabricator hosting service
   429   that is used by the Phabricator hosting service
   430   \<^url>\<open>https://admin.phacility.com\<close>. This avoids various problems with the
   430   \<^url>\<open>https://admin.phacility.com\<close>. This avoids various problems with the
   431   package provided by Ubuntu 18.04 or 20.04. Alternatively, an explicit file
   431   package provided by Ubuntu 20.04. Alternatively, an explicit file path or
   432   path or URL the source archive (\<^verbatim>\<open>.tar.gz\<close>) may be given here. This option
   432   URL the source archive (\<^verbatim>\<open>.tar.gz\<close>) may be given here. This option is
   433   is recommended for production use, but it requires to \<^emph>\<open>uninstall\<close> existing
   433   recommended for production use, but it requires to \<^emph>\<open>uninstall\<close> existing
   434   Mercurial packages provided by the operating system.
   434   Mercurial packages provided by the operating system.
   435 
   435 
   436   Option \<^verbatim>\<open>-n\<close> provides an alternative installation name. The default name
   436   Option \<^verbatim>\<open>-n\<close> provides an alternative installation name. The default name
   437   \<^verbatim>\<open>vcs\<close> means ``version control system''. The name appears in the URL for SSH
   437   \<^verbatim>\<open>vcs\<close> means ``version control system''. The name appears in the URL for SSH
   438   access, and thus has some relevance to end-users. The initial server URL
   438   access, and thus has some relevance to end-users. The initial server URL