src/HOL/TPTP/TPTP_Parser_Example.thy
changeset 47548 60849d8c457d
parent 47518 b2f209258621
child 47558 55b42f9af99d
--- a/src/HOL/TPTP/TPTP_Parser_Example.thy	Wed Apr 18 17:33:11 2012 +0100
+++ b/src/HOL/TPTP/TPTP_Parser_Example.thy	Wed Apr 18 17:33:11 2012 +0100
@@ -9,8 +9,7 @@
 uses "~~/src/HOL/ex/sledgehammer_tactics.ML"
 begin
 
-import_tptp "$TPTP_PROBLEMS_PATH/ALG/ALG001^5.p" (*FIXME multiple imports*)
-(*import_tptp "$TPTP_PROBLEMS_PATH/NUM/NUM021^1.p"*)
+import_tptp "$TPTP_PROBLEMS_PATH/ALG/ALG001^5.p"
 
 ML {*
 val an_fmlas =
@@ -22,7 +21,7 @@
 
 (*Display nicely.*)
 ML {*
-List.app (fn (n, role, _, fmla, _) =>
+List.app (fn (n, role, fmla, _) =>
   Pretty.writeln
     (Pretty.block [Pretty.str ("\"" ^ n ^ "\"" ^ "(" ^
       TPTP_Syntax.role_to_string role  ^ "): "), Syntax.pretty_term @{context} fmla])
@@ -35,9 +34,9 @@
 fun extract_terms roles : TPTP_Interpret.tptp_formula_meaning list ->
  (string * term) list =
    let
-     fun role_predicate (_, role, _, _, _) =
+     fun role_predicate (_, role, _, _) =
        fold (fn r1 => fn b => role = r1 orelse b) roles false
-   in filter role_predicate #> map (fn (n, _, _, t, _) => (n, t)) end
+   in filter role_predicate #> map (fn (n, _, t, _) => (n, t)) end
 *}
 
 ML {*