added map_contexts;
authorwenzelm
Wed, 17 Sep 2008 22:06:57 +0200
changeset 28278 7af26c1f02ec
parent 28277 f2995a28e0e4
child 28279 7d56de7e2305
added map_contexts;
src/Pure/Isar/proof.ML
--- a/src/Pure/Isar/proof.ML	Wed Sep 17 22:06:54 2008 +0200
+++ b/src/Pure/Isar/proof.ML	Wed Sep 17 22:06:57 2008 +0200
@@ -17,6 +17,7 @@
   val context_of: state -> context
   val theory_of: state -> theory
   val map_context: (context -> context) -> state -> state
+  val map_contexts: (context -> context) -> state -> state
   val add_binds_i: (indexname * term option) list -> state -> state
   val put_thms: bool -> string * thm list option -> state -> state
   val the_facts: state -> thm list
@@ -166,6 +167,7 @@
 
 fun current (State st) = Stack.top st |> (fn Node node => node);
 fun map_current f (State st) = State (Stack.map_top (map_node f) st);
+fun map_all f (State st) = State (Stack.map_all (map_node f) st);
 
 
 
@@ -199,6 +201,8 @@
 fun map_context_result f state =
   f (context_of state) ||> (fn ctxt => map_context (K ctxt) state);
 
+fun map_contexts f = map_all (fn (ctxt, facts, mode, goal) => (f ctxt, facts, mode, goal));
+
 val add_binds_i = map_context o ProofContext.add_binds_i;
 val put_thms = map_context oo ProofContext.put_thms;