src/Pure/thm.ML
changeset 70310 c82f59c47aaf
parent 70159 57503fe1b0ff
child 70313 9c19e15c8548
--- a/src/Pure/thm.ML	Mon Jun 03 17:01:28 2019 +0200
+++ b/src/Pure/thm.ML	Mon Jun 03 20:09:43 2019 +0200
@@ -89,6 +89,7 @@
   val transfer: theory -> thm -> thm
   val transfer': Proof.context -> thm -> thm
   val transfer'': Context.generic -> thm -> thm
+  val join_transfer: theory -> thm -> thm
   val renamed_prop: term -> thm -> thm
   val weaken: cterm -> thm -> thm
   val weaken_sorts: sort list -> cterm -> cterm
@@ -530,6 +531,10 @@
 val transfer' = transfer o Proof_Context.theory_of;
 val transfer'' = transfer o Context.theory_of;
 
+fun join_transfer thy th =
+  if Context.subthy_id (Context.theory_id thy, theory_id th) then th
+  else transfer thy th;
+
 
 (* matching *)