clarified ML bootstrap environment;
authorwenzelm
Wed, 06 Apr 2016 14:02:12 +0200
changeset 62887 6b2c60ebd915
parent 62886 72c475e03e22
child 62888 64f44d7279e5
clarified ML bootstrap environment;
src/Pure/ML_Bootstrap.thy
src/Pure/ML_Root.thy
src/Pure/ROOT
src/Pure/ROOT1.ML
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/Pure/ML_Bootstrap.thy	Wed Apr 06 14:02:12 2016 +0200
@@ -0,0 +1,35 @@
+(*  Title:      Pure/ML_Bootstrap.thy
+    Author:     Makarius
+
+ML bootstrap environment -- with access to low-level structures!
+*)
+
+theory ML_Bootstrap
+imports Pure
+keywords "use" "use_debug" "use_no_debug" :: thy_load
+begin
+
+setup \<open>Context.theory_map ML_Env.init_bootstrap\<close>
+
+ML \<open>
+local
+
+val _ =
+  Outer_Syntax.command @{command_keyword use}
+    "read and evaluate Isabelle/ML or SML file"
+    (Resources.parse_files "use" --| @{keyword ";"} >> ML_File.use NONE);
+
+val _ =
+  Outer_Syntax.command @{command_keyword use_debug}
+    "read and evaluate Isabelle/ML or SML file (with debugger information)"
+    (Resources.parse_files "use_debug" --| @{keyword ";"} >> ML_File.use (SOME true));
+
+val _ =
+  Outer_Syntax.command @{command_keyword use_no_debug}
+    "read and evaluate Isabelle/ML or SML file (no debugger information)"
+    (Resources.parse_files "use_no_debug" --| @{keyword ";"} >> ML_File.use (SOME false));
+
+in end
+\<close>
+
+end
--- a/src/Pure/ML_Root.thy	Wed Apr 06 11:57:21 2016 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,35 +0,0 @@
-(*  Title:      Pure/ML_Root.thy
-    Author:     Makarius
-
-Support for ML project ROOT file, with imitation of ML "use" commands.
-*)
-
-theory ML_Root
-imports Pure
-keywords "use" "use_debug" "use_no_debug" :: thy_load
-begin
-
-setup \<open>Context.theory_map ML_Env.init_bootstrap\<close>
-
-ML \<open>
-local
-
-val _ =
-  Outer_Syntax.command @{command_keyword use}
-    "read and evaluate Isabelle/ML or SML file"
-    (Resources.parse_files "use" --| @{keyword ";"} >> ML_File.use NONE);
-
-val _ =
-  Outer_Syntax.command @{command_keyword use_debug}
-    "read and evaluate Isabelle/ML or SML file (with debugger information)"
-    (Resources.parse_files "use_debug" --| @{keyword ";"} >> ML_File.use (SOME true));
-
-val _ =
-  Outer_Syntax.command @{command_keyword use_no_debug}
-    "read and evaluate Isabelle/ML or SML file (no debugger information)"
-    (Resources.parse_files "use_no_debug" --| @{keyword ";"} >> ML_File.use (SOME false));
-
-in end
-\<close>
-
-end
--- a/src/Pure/ROOT	Wed Apr 06 11:57:21 2016 +0200
+++ b/src/Pure/ROOT	Wed Apr 06 14:02:12 2016 +0200
@@ -4,4 +4,4 @@
   global_theories
     Pure
   theories
-    ML_Root
+    ML_Bootstrap
--- a/src/Pure/ROOT1.ML	Wed Apr 06 11:57:21 2016 +0200
+++ b/src/Pure/ROOT1.ML	Wed Apr 06 14:02:12 2016 +0200
@@ -1,6 +1,6 @@
 (*** Isabelle/Pure bootstrap: final setup ***)
 
 use_thy "Pure";
-use_thy "ML_Root";
+use_thy "ML_Bootstrap";
 
 use "ML/ml_pervasive1.ML";