src/HOL/Decision_Procs/cooper_tac.ML
changeset 59621 291934bac95e
parent 59582 0fbed69ff081
child 59629 0d77c51b5040
--- a/src/HOL/Decision_Procs/cooper_tac.ML	Fri Mar 06 14:01:08 2015 +0100
+++ b/src/HOL/Decision_Procs/cooper_tac.ML	Fri Mar 06 15:58:56 2015 +0100
@@ -73,7 +73,7 @@
       |> fold Simplifier.add_cong @{thms conj_le_cong imp_le_cong}
     (* simp rules for elimination of abs *)
     val simpset3 = put_simpset HOL_basic_ss ctxt |> Splitter.add_split @{thm abs_split}
-    val ct = Thm.cterm_of thy (HOLogic.mk_Trueprop t)
+    val ct = Thm.global_cterm_of thy (HOLogic.mk_Trueprop t)
     (* Theorem for the nat --> int transformation *)
     val pre_thm = Seq.hd (EVERY
       [simp_tac mod_div_simpset 1, simp_tac simpset0 1,
@@ -86,7 +86,7 @@
       (case Thm.prop_of pre_thm of
         Const (@{const_name Pure.imp}, _) $ (Const (@{const_name Trueprop}, _) $ t1) $ _ =>
           let
-            val pth = linzqe_oracle (Thm.cterm_of thy (Envir.eta_long [] t1))
+            val pth = linzqe_oracle (Thm.global_cterm_of thy (Envir.eta_long [] t1))
           in
             ((pth RS iffD2) RS pre_thm,
               assm_tac (i + 1) THEN (if q then I else TRY) (rtac TrueI i))