src/Pure/theory.ML
changeset 59930 bdbc4b761c31
parent 58936 7fbe4436952d
child 60099 73c260342704
--- a/src/Pure/theory.ML	Mon Apr 06 12:37:21 2015 +0200
+++ b/src/Pure/theory.ML	Mon Apr 06 12:51:25 2015 +0200
@@ -14,6 +14,7 @@
   val merge: theory * theory -> theory
   val merge_list: theory list -> theory
   val setup: (theory -> theory) -> unit
+  val local_setup: (Proof.context -> Proof.context) -> unit
   val get_markup: theory -> Markup.T
   val axiom_table: theory -> term Name_Space.table
   val axiom_space: theory -> Name_Space.T
@@ -51,6 +52,7 @@
   | merge_list (thy :: thys) = Library.foldl merge (thy, thys);
 
 fun setup f = Context.>> (Context.map_theory f);
+fun local_setup f = Context.>> (Context.map_proof f);