src/Pure/Pure.thy
changeset 68813 78edc4bc3bd3
parent 68505 088780aa2b70
child 68816 5a53724fe247
--- a/src/Pure/Pure.thy	Sun Aug 26 15:39:34 2018 +0200
+++ b/src/Pure/Pure.thy	Sun Aug 26 17:28:38 2018 +0200
@@ -196,10 +196,10 @@
     (Parse.ML_source >> (fn source =>
       Toplevel.generic_theory (fn context =>
         context
-        |> ML_Env.set_bootstrap true
+        |> ML_Env.set_global true
         |> ML_Context.exec (fn () =>
             ML_Context.eval_source (ML_Compiler.verbose true ML_Compiler.flags) source)
-        |> ML_Env.restore_bootstrap context
+        |> ML_Env.restore_global context
         |> Local_Theory.propagate_ml_env)));
 
 val _ =