src/Pure/ML_Bootstrap.thy
author wenzelm
Thu, 07 Apr 2016 21:27:17 +0200
changeset 62910 f37878ebba65
parent 62902 3c0f53eae166
child 62930 51ac6bc389e8
permissions -rw-r--r--
explicit handling of recursive ML name space, e.g. relevant for ML_Bootstrap; handle bootstrap signatures as well;

(*  Title:      Pure/ML_Bootstrap.thy
    Author:     Makarius

ML bootstrap environment -- with access to low-level structures!
*)

theory ML_Bootstrap
imports Pure
begin

setup \<open>Context.theory_map ML_Env.init_bootstrap\<close>
SML_import \<open>structure Thread_Data = Thread_Data_Virtual\<close>
setup \<open>Config.put_global ML_Env.SML_environment true\<close>

end