make sure that enough type information is generated -- because the exported "lemma"s are also used as "conjecture", we can't optimize type information based on polarity
authorblanchet
Tue, 21 Jun 2011 17:17:39 +0200
changeset 43494 13eefebbc4cb
parent 43493 bdb11c68f142
child 43495 75d2e48c5d30
make sure that enough type information is generated -- because the exported "lemma"s are also used as "conjecture", we can't optimize type information based on polarity
src/HOL/ex/atp_export.ML
--- a/src/HOL/ex/atp_export.ML	Tue Jun 21 17:17:39 2011 +0200
+++ b/src/HOL/ex/atp_export.ML	Tue Jun 21 17:17:39 2011 +0200
@@ -8,6 +8,8 @@
 
 signature ATP_EXPORT =
 sig
+  val theorems_mentioned_in_proof_term :
+    string list option -> thm -> string list
   val generate_tptp_graph_file_for_theory :
     Proof.context -> theory -> string -> unit
   val generate_tptp_inference_file_for_theory :
@@ -110,7 +112,7 @@
       facts0 |> map (fn ((_, loc), th) =>
                         ((Thm.get_name_hint th, loc), prop_of th))
     val (atp_problem, _, _, _, _, _, _) =
-      prepare_atp_problem ctxt format Axiom Axiom type_sys false false true []
+      prepare_atp_problem ctxt format Axiom Axiom type_sys true false true []
                           @{prop False} facts
     val all_names = facts0 |> map (Thm.get_name_hint o snd)
     val infers =