src/HOL/Decision_Procs/Commutative_Ring.thy
changeset 67649 1e1782c1aedf
parent 67341 df79ef3b3a41
child 69597 ff784d5a5bfb
--- a/src/HOL/Decision_Procs/Commutative_Ring.thy	Sat Feb 17 20:03:37 2018 +0100
+++ b/src/HOL/Decision_Procs/Commutative_Ring.thy	Sun Feb 18 15:05:21 2018 +0100
@@ -737,7 +737,7 @@
   (case get_matching_rules ctxt (Ring_Simps.get (Context.Proof ctxt)) t of
      SOME (ths1, ths2, ths3, ths4, th5, th) =>
        let val tr =
-         Thm.transfer (Proof_Context.theory_of ctxt) #>
+         Thm.transfer' ctxt #>
          (case optcT of NONE => I | SOME cT => inst [cT] [] #> norm)
        in (map tr ths1, map tr ths2, map tr ths3, map tr ths4, tr th5, tr th) end
    | NONE => error "get_ring_simps: lookup failed");