src/Pure/Isar/local_theory.ML
changeset 49042 01041f7bf9b4
parent 47281 d6c76b1823fb
child 49058 2924a83a4a0b
--- a/src/Pure/Isar/local_theory.ML	Fri Aug 31 15:25:26 2012 +0200
+++ b/src/Pure/Isar/local_theory.ML	Fri Aug 31 16:35:30 2012 +0200
@@ -30,6 +30,8 @@
   val raw_theory: (theory -> theory) -> local_theory -> local_theory
   val background_theory_result: (theory -> 'a * theory) -> local_theory -> 'a * local_theory
   val background_theory: (theory -> theory) -> local_theory -> local_theory
+  val begin_proofs: local_theory -> local_theory
+  val register_proofs: thm list -> local_theory -> local_theory
   val target_of: local_theory -> Proof.context
   val target: (Proof.context -> Proof.context) -> local_theory -> local_theory
   val target_morphism: local_theory -> morphism
@@ -190,6 +192,12 @@
 fun background_theory f = #2 o background_theory_result (f #> pair ());
 
 
+(* forked proofs *)
+
+val begin_proofs = background_theory (Context.theory_map Thm.begin_proofs);
+val register_proofs = background_theory o Context.theory_map o Thm.register_proofs;
+
+
 (* target contexts *)
 
 val target_of = #target o get_last_lthy;