src/Doc/System/Misc.thy
changeset 73150 c9a836122739
parent 72525 8eb0b663fa20
child 73172 fc828f64da5b
equal deleted inserted replaced
73149:bdc8cd6f5e6e 73150:c9a836122739
    69   \<^medskip>
    69   \<^medskip>
    70   Option \<^verbatim>\<open>-B\<close> specifies the Docker image taken as starting point for the
    70   Option \<^verbatim>\<open>-B\<close> specifies the Docker image taken as starting point for the
    71   Isabelle installation: it needs to be a suitable version of Ubuntu Linux.
    71   Isabelle installation: it needs to be a suitable version of Ubuntu Linux.
    72   The default \<^verbatim>\<open>ubuntu\<close> refers to the latest LTS version provided by Canonical
    72   The default \<^verbatim>\<open>ubuntu\<close> refers to the latest LTS version provided by Canonical
    73   as the official Ubuntu vendor\<^footnote>\<open>\<^url>\<open>https://hub.docker.com/_/ubuntu\<close>\<close>. For
    73   as the official Ubuntu vendor\<^footnote>\<open>\<^url>\<open>https://hub.docker.com/_/ubuntu\<close>\<close>. For
    74   Isabelle2020 this should be Ubuntu 18.04 LTS.
    74   Isabelle2021 this should be Ubuntu 20.04 LTS.
    75 
    75 
    76   Option \<^verbatim>\<open>-p\<close> includes additional Ubuntu packages, using the terminology
    76   Option \<^verbatim>\<open>-p\<close> includes additional Ubuntu packages, using the terminology
    77   of \<^verbatim>\<open>apt-get install\<close> within the underlying Linux distribution.
    77   of \<^verbatim>\<open>apt-get install\<close> within the underlying Linux distribution.
    78 
    78 
    79   Option \<^verbatim>\<open>-P\<close> refers to high-level package collections: \<^verbatim>\<open>X11\<close> or \<^verbatim>\<open>latex\<close> as
    79   Option \<^verbatim>\<open>-P\<close> refers to high-level package collections: \<^verbatim>\<open>X11\<close> or \<^verbatim>\<open>latex\<close> as
    96 
    96 
    97 text \<open>
    97 text \<open>
    98   Produce a Dockerfile (without image) from a remote Isabelle distribution:
    98   Produce a Dockerfile (without image) from a remote Isabelle distribution:
    99   @{verbatim [display]
    99   @{verbatim [display]
   100 \<open>  isabelle build_docker -E -n -o Dockerfile
   100 \<open>  isabelle build_docker -E -n -o Dockerfile
   101     https://isabelle.in.tum.de/website-Isabelle2020/dist/Isabelle2020_linux.tar.gz\<close>}
   101     https://isabelle.in.tum.de/website-Isabelle2021/dist/Isabelle2021_linux.tar.gz\<close>}
   102 
   102 
   103   Build a standard Isabelle Docker image from a local Isabelle distribution,
   103   Build a standard Isabelle Docker image from a local Isabelle distribution,
   104   with \<^verbatim>\<open>bin/isabelle\<close> as executable entry point:
   104   with \<^verbatim>\<open>bin/isabelle\<close> as executable entry point:
   105 
   105 
   106   @{verbatim [display]
   106   @{verbatim [display]
   107 \<open>  isabelle build_docker -E -t test/isabelle:Isabelle2020 Isabelle2020_linux.tar.gz\<close>}
   107 \<open>  isabelle build_docker -E -t test/isabelle:Isabelle2021 Isabelle2021_linux.tar.gz\<close>}
   108 
   108 
   109   Invoke the raw Isabelle/ML process within that image:
   109   Invoke the raw Isabelle/ML process within that image:
   110   @{verbatim [display]
   110   @{verbatim [display]
   111 \<open>  docker run test/isabelle:Isabelle2020 process -e "Session.welcome ()"\<close>}
   111 \<open>  docker run test/isabelle:Isabelle2021 process -e "Session.welcome ()"\<close>}
   112 
   112 
   113   Invoke a Linux command-line tool within the contained Isabelle system
   113   Invoke a Linux command-line tool within the contained Isabelle system
   114   environment:
   114   environment:
   115   @{verbatim [display]
   115   @{verbatim [display]
   116 \<open>  docker run test/isabelle:Isabelle2020 env uname -a\<close>}
   116 \<open>  docker run test/isabelle:Isabelle2021 env uname -a\<close>}
   117   The latter should always report a Linux operating system, even when running
   117   The latter should always report a Linux operating system, even when running
   118   on Windows or macOS.
   118   on Windows or macOS.
   119 \<close>
   119 \<close>
   120 
   120 
   121 
   121 
   355 
   355 
   356   Display Isabelle version information.\<close>}
   356   Display Isabelle version information.\<close>}
   357 
   357 
   358   \<^medskip>
   358   \<^medskip>
   359   The default is to output the full version string of the Isabelle
   359   The default is to output the full version string of the Isabelle
   360   distribution, e.g.\ ``\<^verbatim>\<open>Isabelle2020: April 2020\<close>.
   360   distribution, e.g.\ ``\<^verbatim>\<open>Isabelle2021: February 2021\<close>.
   361 
   361 
   362   The \<^verbatim>\<open>-i\<close> option produces a short identification derived from the Mercurial
   362   The \<^verbatim>\<open>-i\<close> option produces a short identification derived from the Mercurial
   363   id of the @{setting ISABELLE_HOME} directory.
   363   id of the @{setting ISABELLE_HOME} directory.
   364 \<close>
   364 \<close>
   365 
   365