src/HOL/Tools/SMT/smt_replay.ML
changeset 70320 59258a3192bf
parent 69593 3dda49e08b9d
child 70749 5d06b7bb9d22
--- a/src/HOL/Tools/SMT/smt_replay.ML	Tue Jun 04 15:14:19 2019 +0200
+++ b/src/HOL/Tools/SMT/smt_replay.ML	Tue Jun 04 15:14:56 2019 +0200
@@ -186,14 +186,14 @@
     |> map (fn ithm as (_, thm) => (ithm, Thm.cprop_of thm aconvc ct))
 in
 
-fun add_asserted tab_update tab_empty p_extract cond outer_ctxt rewrite_rules assms steps ctxt =
+fun add_asserted tab_update tab_empty p_extract cond outer_ctxt rewrite_rules assms steps ctxt0 =
   let
-    val eqs = map (rewrite ctxt [rewrite_true_rule]) rewrite_rules
+    val eqs = map (rewrite ctxt0 [rewrite_true_rule]) rewrite_rules
     val eqs' = union Thm.eq_thm eqs prep_rules
 
     val assms_net =
       assms
-      |> map (apsnd (rewrite ctxt eqs'))
+      |> map (apsnd (rewrite ctxt0 eqs'))
       |> map (apsnd (Conv.fconv_rule Thm.eta_conversion))
       |> thm_net_of snd
 
@@ -229,7 +229,7 @@
         else
           cx
       end
-  in fold add steps (([], []), (ctxt, tab_empty)) end
+  in fold add steps (([], []), (ctxt0, tab_empty)) end
 
 end