src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML
changeset 51208 44f0bfe67b01
parent 51203 4c6ae305462e
child 51212 2bbcc9cc12b4
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Wed Feb 20 16:21:04 2013 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Wed Feb 20 17:05:24 2013 +0100
@@ -678,12 +678,12 @@
                  | _ => NONE)
               | _ => NONE)
         fun dep_of_step (name, _, _, _, from) = SOME (from, name)
+        val bot = atp_proof |> List.last |> dep_of_step |> the |> snd
         val refute_graph =
-          atp_proof |> map_filter dep_of_step |> make_refute_graph
+          atp_proof |> map_filter dep_of_step |> make_refute_graph bot
         val axioms = axioms_of_refute_graph refute_graph conjs
         val tainted = tainted_atoms_of_refute_graph refute_graph conjs
         val is_clause_tainted = exists (member (op =) tainted)
-        val bot = atp_proof |> List.last |> dep_of_step |> the |> snd
         val steps =
           Symtab.empty
           |> fold (fn (name as (s, _), role, t, rule, _) =>