src/HOL/Tools/ATP/atp_translate.ML
changeset 43222 d90151a666cc
parent 43214 4e850b2c1f5c
child 43248 69375eaa9016
--- a/src/HOL/Tools/ATP/atp_translate.ML	Mon Jun 06 23:46:02 2011 +0200
+++ b/src/HOL/Tools/ATP/atp_translate.ML	Tue Jun 07 06:58:52 2011 +0200
@@ -130,7 +130,7 @@
   val prepare_atp_problem :
     Proof.context -> format -> formula_kind -> formula_kind -> type_sys
     -> bool option -> bool -> bool -> term list -> term
-    -> ((string * locality) * thm) list
+    -> ((string * locality) * term) list
     -> string problem * string Symtab.table * int * int
        * (string * locality) list vector * int list * int Symtab.table
   val atp_problem_weights : string problem -> (string * real) list
@@ -1386,10 +1386,10 @@
                        facts =
   let
     val thy = Proof_Context.theory_of ctxt
-    val fact_ts = facts |> map (prop_of o snd)
+    val fact_ts = facts |> map snd
     val (facts, fact_names) =
-      facts |> map (fn (name, th) =>
-                        (name, prop_of th)
+      facts |> map (fn (name, t) =>
+                        (name, t)
                         |> make_fact ctxt format type_sys false true true true
                         |> rpair name)
             |> map_filter (try (apfst the))