updated for release;
authorwenzelm
Tue, 03 Oct 2017 17:35:16 +0200
changeset 66785 6fbd7fc824a9
parent 66687 cd8ad4eddb8a
child 66786 61617dafcd60
updated for release;
src/Doc/System/Environment.thy
src/Doc/System/Misc.thy
src/Pure/Admin/build_docker.scala
--- a/src/Doc/System/Environment.thy	Sat Sep 23 13:46:48 2017 +0200
+++ b/src/Doc/System/Environment.thy	Tue Oct 03 17:35:16 2017 +0200
@@ -141,7 +141,7 @@
   search path of the shell.
 
   \<^descr>[@{setting_def ISABELLE_IDENTIFIER}\<open>\<^sup>*\<close>] refers to the name of this
-  Isabelle distribution, e.g.\ ``\<^verbatim>\<open>Isabelle2012\<close>''.
+  Isabelle distribution, e.g.\ ``\<^verbatim>\<open>Isabelle2017\<close>''.
 
   \<^descr>[@{setting_def ML_SYSTEM}, @{setting_def ML_HOME}, @{setting_def
   ML_OPTIONS}, @{setting_def ML_PLATFORM}, @{setting_def ML_IDENTIFIER}\<open>\<^sup>*\<close>]
--- a/src/Doc/System/Misc.thy	Sat Sep 23 13:46:48 2017 +0200
+++ b/src/Doc/System/Misc.thy	Tue Oct 03 17:35:16 2017 +0200
@@ -220,7 +220,7 @@
 
   \<^medskip>
   The default is to output the full version string of the Isabelle
-  distribution, e.g.\ ``\<^verbatim>\<open>Isabelle2012: May 2012\<close>.
+  distribution, e.g.\ ``\<^verbatim>\<open>Isabelle2017: October 2017\<close>.
 
   The \<^verbatim>\<open>-i\<close> option produces a short identification derived from the Mercurial
   id of the @{setting ISABELLE_HOME} directory.
--- a/src/Pure/Admin/build_docker.scala	Sat Sep 23 13:46:48 2017 +0200
+++ b/src/Pure/Admin/build_docker.scala	Tue Oct 03 17:35:16 2017 +0200
@@ -130,9 +130,9 @@
 
   Examples:
 
-    isabelle build_docker -E -t test/isabelle:Isabelle2016-1 Isabelle2016-1_app.tar.gz
+    isabelle build_docker -E -t test/isabelle:Isabelle2017 Isabelle2017_app.tar.gz
 
-    isabelle build_docker -E -n -o Dockerfile http://isabelle.in.tum.de/dist/Isabelle2016-1_app.tar.gz
+    isabelle build_docker -E -n -o Dockerfile http://isabelle.in.tum.de/dist/Isabelle2017_app.tar.gz
 
 """,
           "B:" -> (arg => base = arg),