src/HOL/Tools/Sledgehammer/sledgehammer_proof_reconstruct.ML
changeset 38738 0ce517c1970f
parent 38698 d19c3a7ce38b
child 38748 69fea359d3f8
equal deleted inserted replaced
38737:bdcb23701448 38738:0ce517c1970f
   232 fun parse_lines pool = Scan.repeat1 (parse_line pool)
   232 fun parse_lines pool = Scan.repeat1 (parse_line pool)
   233 fun parse_proof pool =
   233 fun parse_proof pool =
   234   fst o Scan.finite Symbol.stopper
   234   fst o Scan.finite Symbol.stopper
   235             (Scan.error (!! (fn _ => raise Fail "unrecognized ATP output")
   235             (Scan.error (!! (fn _ => raise Fail "unrecognized ATP output")
   236                             (parse_lines pool)))
   236                             (parse_lines pool)))
   237   o explode o strip_spaces
   237   o explode o strip_spaces_except_between_ident_chars
   238 
   238 
   239 (**** INTERPRETATION OF TSTP SYNTAX TREES ****)
   239 (**** INTERPRETATION OF TSTP SYNTAX TREES ****)
   240 
   240 
   241 exception FO_TERM of string fo_term list
   241 exception FO_TERM of string fo_term list
   242 exception FORMULA of (string, string fo_term) formula list
   242 exception FORMULA of (string, string fo_term) formula list