src/Doc/System/Phabricator.thy
changeset 76010 da54ac51266a
parent 75161 95612f330c93
child 79482 a49db426ffd4
equal deleted inserted replaced
76009:adf9c4d68581 76010:da54ac51266a
    27   standard LAMP server (Linux, Apache, MySQL, PHP). This merely requires a
    27   standard LAMP server (Linux, Apache, MySQL, PHP). This merely requires a
    28   virtual machine on the Net, which can be rented cheaply from local hosting
    28   virtual machine on the Net, which can be rented cheaply from local hosting
    29   providers --- there is no need to follow big cloud corporations. So it is
    29   providers --- there is no need to follow big cloud corporations. So it is
    30   feasible to remain the master of your virtual home, following the slogan
    30   feasible to remain the master of your virtual home, following the slogan
    31   ``own all your data''. In many respects, Phabricator is similar to the
    31   ``own all your data''. In many respects, Phabricator is similar to the
    32   well-known Nextcloud\<^footnote>\<open>\<^url>\<open>https://nextcloud.org\<close>\<close> product, concerning both
    32   well-known Nextcloud\<^footnote>\<open>\<^url>\<open>https://nextcloud.com\<close>\<close> product, concerning both
    33   the technology and sociology.
    33   the technology and sociology.
    34 
    34 
    35   \<^medskip>
    35   \<^medskip>
    36   The following Phabricator instances may serve as examples:
    36   The following Phabricator instances may serve as examples:
    37 
    37 
    38     \<^item> Phabricator development \<^url>\<open>https://secure.phabricator.com\<close>
       
    39     \<^item> Wikimedia development \<^url>\<open>https://phabricator.wikimedia.org\<close>
    38     \<^item> Wikimedia development \<^url>\<open>https://phabricator.wikimedia.org\<close>
    40     \<^item> Blender development \<^url>\<open>https://developer.blender.org\<close>
    39     \<^item> Blender development \<^url>\<open>https://developer.blender.org\<close>
    41     \<^item> LLVM development \<^url>\<open>https://reviews.llvm.org\<close>
    40     \<^item> LLVM development \<^url>\<open>https://reviews.llvm.org\<close>
    42     \<^item> Mozilla development \<^url>\<open>https://phabricator.services.mozilla.com\<close>
    41     \<^item> Mozilla development \<^url>\<open>https://phabricator.services.mozilla.com\<close>
    43     \<^item> Mercurial development \<^url>\<open>https://phab.mercurial-scm.org\<close>
       
    44     \<^item> Isabelle development \<^url>\<open>https://isabelle-dev.sketis.net\<close>
    42     \<^item> Isabelle development \<^url>\<open>https://isabelle-dev.sketis.net\<close>
       
    43     \<^item> Phabricator development (inactive) \<^url>\<open>https://secure.phabricator.com\<close>
       
    44     \<^item> Phorge development (planned successor of Phabricator)
       
    45       \<^url>\<open>https://we.phorge.it\<close>
    45 
    46 
    46   \<^medskip>
    47   \<^medskip>
    47   Initial Phabricator configuration requires many details to be done right.
    48   Initial Phabricator configuration requires many details to be done right.
    48   Isabelle provides some command-line tools to help with the setup, and
    49   Isabelle provides some command-line tools to help with the setup, and
    49   afterwards Isabelle support is optional: it is possible to run and maintain
    50   afterwards Isabelle support is optional: it is possible to run and maintain
   232     Then reload (or restart) Apache like this:
   233     Then reload (or restart) Apache like this:
   233     @{verbatim [display] \<open>  systemctl reload apache2\<close>}
   234     @{verbatim [display] \<open>  systemctl reload apache2\<close>}
   234 
   235 
   235     \<^item> Install \<^verbatim>\<open>certbot\<close> from \<^url>\<open>https://certbot.eff.org\<close> following the
   236     \<^item> Install \<^verbatim>\<open>certbot\<close> from \<^url>\<open>https://certbot.eff.org\<close> following the
   236     description for Apache and Ubuntu 20.04 on
   237     description for Apache and Ubuntu 20.04 on
   237     \<^url>\<open>https://certbot.eff.org/lets-encrypt/ubuntubionic-apache\<close>. Run
   238     \<^url>\<open>https://certbot.eff.org/instructions?ws=apache&os=ubuntufocal\<close>. Run
   238     \<^verbatim>\<open>certbot\<close> interactively and let it operate on the domain
   239     \<^verbatim>\<open>certbot\<close> interactively and let it operate on the domain
   239     \<^verbatim>\<open>vcs.example.org\<close>.
   240     \<^verbatim>\<open>vcs.example.org\<close>.
   240 
   241 
   241     \<^item> Inform Phabricator about its new domain name like this:
   242     \<^item> Inform Phabricator about its new domain name like this:
   242     @{verbatim [display] \<open>  isabelle phabricator bin/config set \
   243     @{verbatim [display] \<open>  isabelle phabricator bin/config set \