src/Doc/System/Phabricator.thy
changeset 71296 71ea54e851ad
parent 71295 6aadbd650280
child 71322 0256ce61f405
equal deleted inserted replaced
71295:6aadbd650280 71296:71ea54e851ad
    39     \<^item> Wikimedia development \<^url>\<open>https://phabricator.wikimedia.org\<close>
    39     \<^item> Wikimedia development \<^url>\<open>https://phabricator.wikimedia.org\<close>
    40     \<^item> Blender development \<^url>\<open>https://developer.blender.org\<close>
    40     \<^item> Blender development \<^url>\<open>https://developer.blender.org\<close>
    41     \<^item> Mercurial development \<^url>\<open>https://phab.mercurial-scm.org\<close>
    41     \<^item> Mercurial development \<^url>\<open>https://phab.mercurial-scm.org\<close>
    42     \<^item> Isabelle development \<^url>\<open>https://isabelle-dev.sketis.net\<close>
    42     \<^item> Isabelle development \<^url>\<open>https://isabelle-dev.sketis.net\<close>
    43 
    43 
    44   \<^medskip> Initial Phabricator configuration requires many details to be done
    44   \<^medskip>
    45   right.\<^footnote>\<open>See also
    45   Initial Phabricator configuration requires many details to be done right.
    46   \<^url>\<open>https://secure.phabricator.com/book/phabricator/article/installation_guide\<close>
    46   Isabelle provides some command-line tools to help with the setup, and
    47   in the context of \<^url>\<open>https://help.ubuntu.com/lts/serverguide\<close>.\<close> Isabelle
    47   afterwards Isabelle support is optional: it is possible to run and maintain
    48   provides some command-line tools to help with the setup, and afterwards
    48   the server, without requiring the somewhat bulky Isabelle distribution
    49   Isabelle support is optional: it is possible to run and maintain the server,
    49   again.
    50   without requiring the somewhat bulky Isabelle distribution again.
       
    51 \<close>
    50 \<close>
    52 
    51 
    53 
    52 
    54 section \<open>Quick start\<close>
    53 section \<open>Quick start\<close>
    55 
    54 
   243       \<^item> Enable \<^verbatim>\<open>policy.allow-public\<close> to allow read-only access to resources,
   242       \<^item> Enable \<^verbatim>\<open>policy.allow-public\<close> to allow read-only access to resources,
   244       without requiring user registration.
   243       without requiring user registration.
   245 \<close>
   244 \<close>
   246 
   245 
   247 
   246 
   248 section \<open>Global data storage and backups\<close>
   247 section \<open>Global data storage and backups \label{sec:phabricator-backup}\<close>
   249 
   248 
   250 text \<open>
   249 text \<open>
   251   The global state of a Phabricator installation consists of two main parts:
   250   The global state of a Phabricator installation consists of two main parts:
   252 
   251 
   253     \<^enum> The \<^emph>\<open>root directory\<close> according to
   252     \<^enum> The \<^emph>\<open>root directory\<close> according to
   295 
   294 
   296 text \<open>
   295 text \<open>
   297   The Phabricator developers publish a new version approx.\ every 1--4 weeks:
   296   The Phabricator developers publish a new version approx.\ every 1--4 weeks:
   298   see also \<^url>\<open>https://secure.phabricator.com/w/changelog\<close>. There is no need to
   297   see also \<^url>\<open>https://secure.phabricator.com/w/changelog\<close>. There is no need to
   299   follow such frequent updates on the spot, but it is a good idea to upgrade
   298   follow such frequent updates on the spot, but it is a good idea to upgrade
   300   occasionally, see also
   299   occasionally --- after dump and/or backup (\secref{sec:phabricator-backup}).
   301   \<^url>\<open>https://secure.phabricator.com/book/phabricator/article/upgrading\<close> for
       
   302   general explanations.
       
   303 
   300 
   304   The Isabelle/Phabricator setup provides a convenience tool to upgrade all
   301   The Isabelle/Phabricator setup provides a convenience tool to upgrade all
   305   installations uniformly:
   302   installations uniformly:
   306   @{verbatim [display] \<open>  /usr/local/bin/isabelle-phabricator-upgrade\<close>}
   303   @{verbatim [display] \<open>  /usr/local/bin/isabelle-phabricator-upgrade\<close>}
   307 
   304 
   308   This refers to the \<^verbatim>\<open>stable\<close> branch of the distribution repositories by
   305   This refers to the \<^verbatim>\<open>stable\<close> branch of the distribution repositories by
   309   default. Alternatively, it also possible to use the \<^verbatim>\<open>master\<close> like this:
   306   default. Alternatively, it also possible to use the \<^verbatim>\<open>master\<close> like this:
   310   @{verbatim [display] \<open>  /usr/local/bin/isabelle-phabricator-upgrade master\<close>}
   307   @{verbatim [display] \<open>  /usr/local/bin/isabelle-phabricator-upgrade master\<close>}
       
   308 
       
   309   \<^medskip>
       
   310   See
       
   311   \<^url>\<open>https://secure.phabricator.com/book/phabricator/article/upgrading\<close> for
       
   312   further explanations on Phabricator upgrade.
   311 \<close>
   313 \<close>
   312 
   314 
   313 
   315 
   314 section \<open>Reference of command-line tools\<close>
   316 section \<open>Reference of command-line tools\<close>
   315 
   317