src/HOL/Tools/ATP/atp_proof.ML
changeset 43246 01b6391a763f
parent 43163 31babd4b1552
child 43465 5ca37e764139
equal deleted inserted replaced
43245:cef69d31bfa4 43246:01b6391a763f
   197 fun extract_tstplike_proof_and_outcome verbose complete res_code proof_delims
   197 fun extract_tstplike_proof_and_outcome verbose complete res_code proof_delims
   198                                        known_failures output =
   198                                        known_failures output =
   199   case (extract_tstplike_proof proof_delims output,
   199   case (extract_tstplike_proof proof_delims output,
   200         extract_known_failure known_failures output) of
   200         extract_known_failure known_failures output) of
   201     (_, SOME ProofIncomplete) => ("", SOME ProofIncomplete)
   201     (_, SOME ProofIncomplete) => ("", SOME ProofIncomplete)
       
   202   | ("", SOME ProofMissing) => ("", NONE)
   202   | ("", SOME failure) =>
   203   | ("", SOME failure) =>
   203     ("", SOME (if failure = GaveUp andalso complete then Unprovable
   204     ("", SOME (if failure = GaveUp andalso complete then Unprovable
   204                else failure))
   205                else failure))
   205   | ("", NONE) =>
   206   | ("", NONE) => ("", SOME (UnknownError (short_output verbose output)))
   206     ("", SOME (if res_code = 0 andalso output = "" then ProofMissing
       
   207                else UnknownError (short_output verbose output)))
       
   208   | (tstplike_proof, _) => (tstplike_proof, NONE)
   207   | (tstplike_proof, _) => (tstplike_proof, NONE)
   209 
   208 
   210 type step_name = string * string option
   209 type step_name = string * string option
   211 
   210 
   212 fun is_same_atp_step (s1, _) (s2, _) = s1 = s2
   211 fun is_same_atp_step (s1, _) (s2, _) = s1 = s2