src/HOL/Tools/SMT2/z3_new_replay.ML
changeset 57220 853557cf2efa
parent 57219 34018603e0d0
child 57229 489083abce44
--- a/src/HOL/Tools/SMT2/z3_new_replay.ML	Wed Jun 11 19:15:54 2014 +0200
+++ b/src/HOL/Tools/SMT2/z3_new_replay.ML	Wed Jun 11 19:15:55 2014 +0200
@@ -58,7 +58,7 @@
 
 fun replay_thm ctxt assumed nthms
     (Z3_New_Proof.Z3_Step {id, rule, concl, fixes, is_fix_step, ...}) =
-  if Z3_New_Replay_Methods.is_assumption rule then
+  if Z3_New_Proof.is_assumption rule then
     (case Inttab.lookup assumed id of
       SOME (_, thm) => thm
     | NONE => Thm.assume (SMT2_Util.certify ctxt concl))
@@ -115,7 +115,7 @@
 
     fun add (Z3_New_Proof.Z3_Step {id, rule, concl, fixes, ...})
         (cx as ((iidths, thms), (ctxt, ptab))) =
-      if Z3_New_Replay_Methods.is_assumption rule andalso rule <> Z3_New_Proof.Hypothesis then
+      if Z3_New_Proof.is_assumption rule andalso rule <> Z3_New_Proof.Hypothesis then
         let
           val ct = SMT2_Util.certify ctxt concl
           val thm1 = Thm.trivial ct |> Conv.fconv_rule (Conv.arg1_conv (revert_conv outer_ctxt))