diff -r 6aadbd650280 -r 71ea54e851ad src/Doc/System/Phabricator.thy --- a/src/Doc/System/Phabricator.thy Tue Dec 17 13:35:03 2019 +0100 +++ b/src/Doc/System/Phabricator.thy Tue Dec 17 13:43:31 2019 +0100 @@ -41,13 +41,12 @@ \<^item> Mercurial development \<^url>\https://phab.mercurial-scm.org\ \<^item> Isabelle development \<^url>\https://isabelle-dev.sketis.net\ - \<^medskip> Initial Phabricator configuration requires many details to be done - right.\<^footnote>\See also - \<^url>\https://secure.phabricator.com/book/phabricator/article/installation_guide\ - in the context of \<^url>\https://help.ubuntu.com/lts/serverguide\.\ Isabelle - provides some command-line tools to help with the setup, and afterwards - Isabelle support is optional: it is possible to run and maintain the server, - without requiring the somewhat bulky Isabelle distribution again. + \<^medskip> + Initial Phabricator configuration requires many details to be done right. + Isabelle provides some command-line tools to help with the setup, and + afterwards Isabelle support is optional: it is possible to run and maintain + the server, without requiring the somewhat bulky Isabelle distribution + again. \ @@ -245,7 +244,7 @@ \ -section \Global data storage and backups\ +section \Global data storage and backups \label{sec:phabricator-backup}\ text \ The global state of a Phabricator installation consists of two main parts: @@ -297,9 +296,7 @@ The Phabricator developers publish a new version approx.\ every 1--4 weeks: see also \<^url>\https://secure.phabricator.com/w/changelog\. There is no need to follow such frequent updates on the spot, but it is a good idea to upgrade - occasionally, see also - \<^url>\https://secure.phabricator.com/book/phabricator/article/upgrading\ for - general explanations. + occasionally --- after dump and/or backup (\secref{sec:phabricator-backup}). The Isabelle/Phabricator setup provides a convenience tool to upgrade all installations uniformly: @@ -308,6 +305,11 @@ This refers to the \<^verbatim>\stable\ branch of the distribution repositories by default. Alternatively, it also possible to use the \<^verbatim>\master\ like this: @{verbatim [display] \ /usr/local/bin/isabelle-phabricator-upgrade master\} + + \<^medskip> + See + \<^url>\https://secure.phabricator.com/book/phabricator/article/upgrading\ for + further explanations on Phabricator upgrade. \