src/HOL/Tools/ATP_Manager/atp_systems.ML
changeset 37996 11c076ea92e9
parent 37995 06f02b15ef8a
child 37997 abf8a79853c9
--- a/src/HOL/Tools/ATP_Manager/atp_systems.ML	Mon Jul 26 17:03:21 2010 +0200
+++ b/src/HOL/Tools/ATP_Manager/atp_systems.ML	Mon Jul 26 17:09:10 2010 +0200
@@ -287,8 +287,7 @@
                                               thm_names =
   if String.isSubstring set_ClauseFormulaRelationN output then
     let
-      (* FIXME: hd of head once clausification is left to the ATP *)
-      val j0 = hd (List.concat conjecture_shape)
+      val j0 = hd conjecture_shape
       val seq = extract_clause_sequence output
       val name_map = extract_clause_formula_relation output
       fun renumber_conjecture j =
@@ -296,7 +295,7 @@
         |> the_single
         |> (fn s => find_index (curry (op =) s) seq + 1)
     in
-      (conjecture_shape |> map (map renumber_conjecture),
+      (conjecture_shape |> map renumber_conjecture,
        seq |> map (the o AList.lookup (op =) name_map)
            |> map (fn s => case try (unprefix axiom_prefix) s of
                              SOME s' => undo_ascii_of s'
@@ -404,7 +403,6 @@
                             explicit_apply probfile clauses
           val conjecture_shape =
             conjecture_offset + 1 upto conjecture_offset + length hyp_ts + 1
-            |> map single (* ### FIXME: get rid of "map single" *)
           val result =
             do_run false
             |> (fn (_, msecs0, _, SOME _) =>