src/Doc/System/Phabricator.thy
changeset 71322 0256ce61f405
parent 71296 71ea54e851ad
child 71323 7c27a379190f
equal deleted inserted replaced
71321:edf3210a61a2 71322:0256ce61f405
     2 
     2 
     3 theory Phabricator
     3 theory Phabricator
     4 imports Base
     4 imports Base
     5 begin
     5 begin
     6 
     6 
     7 chapter \<open>Phabricator server administration\<close>
     7 chapter \<open>Phabricator server setup \label{ch:phabricator}\<close>
     8 
     8 
     9 text \<open>
     9 text \<open>
    10   Phabricator\<^footnote>\<open>\<^url>\<open>https://www.phacility.com/phabricator\<close>\<close> is an open-source
    10   Phabricator\<^footnote>\<open>\<^url>\<open>https://www.phacility.com/phabricator\<close>\<close> is an open-source
    11   product to support the development process of complex software projects
    11   product to support the development process of complex software projects
    12   (open or closed ones). The official slogan is:
    12   (open or closed ones). The official slogan is:
    45   Initial Phabricator configuration requires many details to be done right.
    45   Initial Phabricator configuration requires many details to be done right.
    46   Isabelle provides some command-line tools to help with the setup, and
    46   Isabelle provides some command-line tools to help with the setup, and
    47   afterwards Isabelle support is optional: it is possible to run and maintain
    47   afterwards Isabelle support is optional: it is possible to run and maintain
    48   the server, without requiring the somewhat bulky Isabelle distribution
    48   the server, without requiring the somewhat bulky Isabelle distribution
    49   again.
    49   again.
       
    50 
       
    51   \<^medskip>
       
    52   Assuming an existing Phabricator installation, the command-line tool @{tool
       
    53   hg_setup} (\secref{sec:hg-setup}) helps to create new repositories or to
       
    54   migrate old ones. In particular, this avoids the lengthy sequence of clicks
       
    55   in Phabricator to make a new private repository with hosting on the server.
       
    56   (Phabricator is a software project management platform, where initial
       
    57   repository setup happens rarely in practice.)
    50 \<close>
    58 \<close>
    51 
    59 
    52 
    60 
    53 section \<open>Quick start\<close>
    61 section \<open>Quick start\<close>
    54 
    62