src/Pure/ML/ml_context.ML
changeset 39911 2b4430847310
parent 39796 b5f978f97347
child 41375 7a89b4b94817
--- a/src/Pure/ML/ml_context.ML	Fri Oct 01 16:05:25 2010 +0200
+++ b/src/Pure/ML/ml_context.ML	Fri Oct 01 17:06:49 2010 +0200
@@ -36,9 +36,6 @@
   val eval_text_in: Proof.context option -> bool -> Position.T -> Symbol_Pos.text -> unit
   val expression: Position.T -> string -> string -> ML_Lex.token Antiquote.antiquote list ->
     Context.generic -> Context.generic
-  val value: Proof.context ->
-    (Proof.context -> unit -> 'a) * ((unit -> 'a) -> Proof.context -> Proof.context) * string ->
-    string * string -> 'a
 end
 
 structure ML_Context: ML_CONTEXT =
@@ -215,17 +212,6 @@
     (ML_Lex.read Position.none ("Context.set_thread_data (SOME (let " ^ bind ^ " = ") @ ants @
       ML_Lex.read Position.none (" in " ^ body ^ " end (ML_Context.the_generic_context ())));")));
 
-fun value ctxt (get, put, put_ml) (prelude, value) =
-  let
-    val code = (prelude
-      ^ "\nval _ = Context.set_thread_data (SOME (Context.map_proof (" ^ put_ml
-      ^ " (fn () => " ^ value ^ ")) (ML_Context.the_generic_context ())))");
-    val ctxt' = ctxt
-      |> put (fn () => error ("Bad evaluation for " ^ quote put_ml))
-      |> Context.proof_map (exec
-          (fn () => Secure.use_text ML_Env.local_context (0, "value") false code));
-  in get ctxt' () end;
-
 end;
 
 structure Basic_ML_Context: BASIC_ML_CONTEXT = ML_Context;