src/HOL/Tools/ATP/atp_util.ML
changeset 59582 0fbed69ff081
parent 59433 9da5b2c61049
child 59621 291934bac95e
--- a/src/HOL/Tools/ATP/atp_util.ML	Tue Mar 03 19:08:04 2015 +0100
+++ b/src/HOL/Tools/ATP/atp_util.ML	Wed Mar 04 19:53:18 2015 +0100
@@ -342,7 +342,7 @@
   if exists_Const (fn (s, _) => s = @{const_name Not}) t then
     t |> Skip_Proof.make_thm thy
       |> Meson.cong_extensionalize_thm thy
-      |> prop_of
+      |> Thm.prop_of
   else
     t
 
@@ -353,8 +353,8 @@
 fun abs_extensionalize_term ctxt t =
   if exists_Const is_fun_equality t then
     let val thy = Proof_Context.theory_of ctxt in
-      t |> cterm_of thy |> Meson.abs_extensionalize_conv ctxt
-        |> prop_of |> Logic.dest_equals |> snd
+      t |> Thm.cterm_of thy |> Meson.abs_extensionalize_conv ctxt
+        |> Thm.prop_of |> Logic.dest_equals |> snd
     end
   else
     t
@@ -405,7 +405,7 @@
 fun strip_subgoal goal i ctxt =
   let
     val (t, (frees, params)) =
-      Logic.goal_params (prop_of goal) i
+      Logic.goal_params (Thm.prop_of goal) i
       ||> (map dest_Free #> Variable.variant_frees ctxt [] #> `(map Free))
     val hyp_ts = t |> Logic.strip_assums_hyp |> map (curry subst_bounds frees)
     val concl_t = t |> Logic.strip_assums_concl |> curry subst_bounds frees