compile
authorblanchet
Tue, 22 May 2012 16:59:27 +0200
changeset 47957 d2bdd85ee23c
parent 47956 2a420750248b
child 47958 c5f7be4a1734
compile
src/HOL/TPTP/atp_problem_import.ML
--- a/src/HOL/TPTP/atp_problem_import.ML	Tue May 22 16:59:27 2012 +0200
+++ b/src/HOL/TPTP/atp_problem_import.ML	Tue May 22 16:59:27 2012 +0200
@@ -75,7 +75,7 @@
   let
     val (conjs, (defs, nondefs), ctxt) = read_tptp_file thy I file_name
     val thy = Proof_Context.theory_of ctxt
-    val defs = defs |> map (ATP_Util.extensionalize_term ctxt
+    val defs = defs |> map (ATP_Util.abs_extensionalize_term ctxt
                             #> aptrueprop (open_form I))
     val state = Proof.init ctxt
     val params =