src/Doc/System/Phabricator.thy
changeset 71286 058edb8f232c
parent 71280 5a2033fc8f3d
child 71290 8d21cba3bad4
equal deleted inserted replaced
71285:8cd05f7b3b4a 71286:058edb8f232c
   288   @{verbatim [display] \<open>  phabricator/bin/repository help list-paths
   288   @{verbatim [display] \<open>  phabricator/bin/repository help list-paths
   289   phabricator/bin/repository help move-paths\<close>}
   289   phabricator/bin/repository help move-paths\<close>}
   290 \<close>
   290 \<close>
   291 
   291 
   292 
   292 
       
   293 section \<open>Upgrading Phabricator installations\<close>
       
   294 
       
   295 text \<open>
       
   296   The Phabricator developers publish a new version approx.\ every 1--4 weeks:
       
   297   see also \<^url>\<open>https://secure.phabricator.com/w/changelog\<close>. There is no need to
       
   298   follow such frequent updates on the spot, but it is a good idea to upgrade
       
   299   occasionally, see also
       
   300   \<^url>\<open>https://secure.phabricator.com/book/phabricator/article/upgrading\<close> for
       
   301   general explanations.
       
   302 
       
   303   The Isabelle/Phabricator setup provides a convenience tool to upgrade all
       
   304   installations uniformly:
       
   305   @{verbatim [display] \<open>  /usr/local/bin/isabelle-phabricator-upgrade\<close>}
       
   306 
       
   307   This refers to the \<^verbatim>\<open>stable\<close> branch of the distribution repositories by
       
   308   default. Alternatively, it also possible to use the \<^verbatim>\<open>master\<close> like this:
       
   309   @{verbatim [display] \<open>  /usr/local/bin/isabelle-phabricator-upgrade master\<close>}
       
   310 \<close>
       
   311 
       
   312 
   293 section \<open>Reference of command-line tools\<close>
   313 section \<open>Reference of command-line tools\<close>
   294 
   314 
   295 text \<open>
   315 text \<open>
   296   The subsequent command-line tools usually require root user privileges on
   316   The subsequent command-line tools usually require root user privileges on
   297   the underlying Linux system (e.g.\ via \<^verbatim>\<open>sudo bash\<close> to open a subshell, or
   317   the underlying Linux system (e.g.\ via \<^verbatim>\<open>sudo bash\<close> to open a subshell, or