src/HOL/Tools/ATP/atp_problem_generate.ML
changeset 57547 677b07d777c3
parent 57541 147e3f1e0459
child 58200 d95055489fce
--- a/src/HOL/Tools/ATP/atp_problem_generate.ML	Sat Jul 12 11:31:22 2014 +0200
+++ b/src/HOL/Tools/ATP/atp_problem_generate.ML	Sat Jul 12 11:31:23 2014 +0200
@@ -1275,30 +1275,17 @@
     {name = name, stature = stature, role = role, iformula = iformula, atomic_types = atomic_Ts}
   end
 
-fun is_format_with_defs (THF _) = true
-  | is_format_with_defs _ = false
-
-fun make_fact ctxt format type_enc iff_for_eq ((name, stature as (_, status)), t) =
-  let
-    val role =
-      if is_format_with_defs format andalso status = Non_Rec_Def andalso
-         is_legitimate_tptp_def t then
-        Definition
-      else
-        Axiom
-  in
-    (case make_formula ctxt format type_enc iff_for_eq name stature role t of
-      formula as {iformula = AAtom (IConst ((s, _), _, _)), ...} =>
-      if s = tptp_true then NONE else SOME formula
-    | formula => SOME formula)
-  end
+fun make_fact ctxt format type_enc iff_for_eq ((name, stature), t) =
+  (case make_formula ctxt format type_enc iff_for_eq name stature Axiom t of
+    formula as {iformula = AAtom (IConst ((s, _), _, _)), ...} =>
+    if s = tptp_true then NONE else SOME formula
+  | formula => SOME formula)
 
 fun make_conjecture ctxt format type_enc =
   map (fn ((name, stature), (role, t)) =>
-    let
-      val role' = if role <> Conjecture andalso is_legitimate_tptp_def t then Definition else role
-      val t' = t |> role' = Conjecture ? s_not
-    in make_formula ctxt format type_enc true name stature role' t' end)
+    let val t' = t |> role = Conjecture ? s_not in
+      make_formula ctxt format type_enc true name stature role t'
+    end)
 
 (** Finite and infinite type inference **)