src/Pure/more_thm.ML
changeset 49058 2924a83a4a0b
parent 49011 9c68e43502ce
child 49062 7e31dfd99ce7
--- a/src/Pure/more_thm.ML	Fri Aug 31 16:35:30 2012 +0200
+++ b/src/Pure/more_thm.ML	Fri Aug 31 22:24:14 2012 +0200
@@ -96,6 +96,7 @@
   val kind_rule: string -> thm -> thm
   val kind: string -> attribute
   val register_proofs: thm list -> Context.generic -> Context.generic
+  val register_proofs_thy: thm list -> theory -> theory
   val begin_proofs: Context.generic -> Context.generic
   val join_local_proofs: Proof.context -> unit
   val join_recent_proofs: theory -> unit
@@ -493,6 +494,7 @@
 
 val begin_proofs = Proofs.map (apfst (K empty_proofs));
 val register_proofs = Proofs.map o pairself o add_proofs;
+val register_proofs_thy = Context.theory_map o register_proofs;
 
 val join_local_proofs = force_proofs o #1 o Proofs.get o Context.Proof;
 val join_recent_proofs = force_proofs o #1 o Proofs.get o Context.Theory;