src/Doc/System/Phabricator.thy
changeset 72519 f760554a5a29
parent 71422 5d5be87330b5
child 72521 354bfab78cbf
equal deleted inserted replaced
72518:4be6ae020fc4 72519:f760554a5a29
    71   For production use, a proper \<^emph>\<open>Virtual Server\<close> or \<^emph>\<open>Root Server\<close> product
    71   For production use, a proper \<^emph>\<open>Virtual Server\<close> or \<^emph>\<open>Root Server\<close> product
    72   from a hosting provider will be required, including an Internet Domain Name
    72   from a hosting provider will be required, including an Internet Domain Name
    73   (\secref{sec:phabricator-domain}).
    73   (\secref{sec:phabricator-domain}).
    74 
    74 
    75   Initial experimentation also works on a local host, e.g.\ via
    75   Initial experimentation also works on a local host, e.g.\ via
    76   VirtualBox\<^footnote>\<open>\<^url>\<open>https://www.virtualbox.org\<close>\<close>. The public domain \<^verbatim>\<open>lvh.me\<close> is
    76   VirtualBox\<^footnote>\<open>\<^url>\<open>https://www.virtualbox.org\<close>\<close>. The Internet domain \<^verbatim>\<open>lvh.me\<close>
    77   used by default: it maps arbitrary subdomains to \<^verbatim>\<open>localhost\<close>.
    77   is used by default: it maps arbitrary subdomains to \<^verbatim>\<open>localhost\<close>.
    78 
    78 
    79   All administrative commands need to be run as \<^verbatim>\<open>root\<close> user (e.g.\ via
    79   All administrative commands need to be run as \<^verbatim>\<open>root\<close> user (e.g.\ via
    80   \<^verbatim>\<open>sudo\<close>). Note that Isabelle refers to user-specific configuration in the
    80   \<^verbatim>\<open>sudo\<close>). Note that Isabelle refers to user-specific configuration in the
    81   user home directory via @{setting ISABELLE_HOME_USER}
    81   user home directory via @{setting ISABELLE_HOME_USER}
    82   (\secref{sec:settings}); that may be different or absent for the root user
    82   (\secref{sec:settings}); that may be different or absent for the root user
   210   The tool can be invoked multiple times with different parameters; ports are
   210   The tool can be invoked multiple times with different parameters; ports are
   211   changed back and forth each time and services restarted.
   211   changed back and forth each time and services restarted.
   212 \<close>
   212 \<close>
   213 
   213 
   214 
   214 
   215 subsection \<open>Public domain name and HTTPS configuration \label{sec:phabricator-domain}\<close>
   215 subsection \<open>Internet domain name and HTTPS configuration \label{sec:phabricator-domain}\<close>
   216 
   216 
   217 text \<open>
   217 text \<open>
   218   So far the Phabricator server has been accessible only on \<^verbatim>\<open>localhost\<close> (via
   218   So far the Phabricator server has been accessible only on \<^verbatim>\<open>localhost\<close> (via
   219   the alias \<^verbatim>\<open>lvh.me\<close>). Proper configuration of a public Internet domain name
   219   the alias \<^verbatim>\<open>lvh.me\<close>). Proper configuration of a public Internet domain name
   220   (with HTTPS certificate from \<^emph>\<open>Let's Encrypt\<close>) works as follows.
   220   (with HTTPS certificate from \<^emph>\<open>Let's Encrypt\<close>) works as follows.