src/Pure/Pure.thy
changeset 68827 1286ca9dfd26
parent 68826 deefe5837120
child 68876 cefaac3d24ff
equal deleted inserted replaced
68826:deefe5837120 68827:1286ca9dfd26
   198         context
   198         context
   199         |> Config.put_generic ML_Env.ML_environment ML_Env.Isabelle
   199         |> Config.put_generic ML_Env.ML_environment ML_Env.Isabelle
   200         |> Config.put_generic ML_Env.ML_write_global true
   200         |> Config.put_generic ML_Env.ML_write_global true
   201         |> ML_Context.exec (fn () =>
   201         |> ML_Context.exec (fn () =>
   202             ML_Context.eval_source (ML_Compiler.verbose true ML_Compiler.flags) source)
   202             ML_Context.eval_source (ML_Compiler.verbose true ML_Compiler.flags) source)
   203         |> Config.put_generic ML_Env.ML_write_global
   203         |> Config.restore_generic ML_Env.ML_write_global context
   204             (Config.get_generic context ML_Env.ML_write_global)
   204         |> Config.restore_generic ML_Env.ML_environment context
   205         |> Config.put_generic ML_Env.ML_environment
       
   206             (Config.get_generic context ML_Env.ML_environment)
       
   207         |> Local_Theory.propagate_ml_env)));
   205         |> Local_Theory.propagate_ml_env)));
   208 
   206 
   209 val _ =
   207 val _ =
   210   Outer_Syntax.command \<^command_keyword>\<open>ML_prf\<close> "ML text within proof"
   208   Outer_Syntax.command \<^command_keyword>\<open>ML_prf\<close> "ML text within proof"
   211     (Parse.ML_source >> (fn source =>
   209     (Parse.ML_source >> (fn source =>