src/Pure/ML_Bootstrap.thy
changeset 67105 05ff3e6dbbce
parent 64331 abf7b6e6865f
child 67147 dea94b1aabc3
--- a/src/Pure/ML_Bootstrap.thy	Tue Nov 28 22:14:10 2017 +0100
+++ b/src/Pure/ML_Bootstrap.thy	Wed Nov 29 10:27:56 2017 +0100
@@ -8,6 +8,9 @@
 imports Pure
 begin
 
+external_file "$POLYML_EXE"
+
+
 subsection \<open>Standard ML environment for virtual bootstrap\<close>
 
 setup \<open>Context.theory_map ML_Env.init_bootstrap\<close>