src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
changeset 56093 4eeb73a1feec
parent 56081 72fad75baf7e
child 56097 8e7a9ad44e14
equal deleted inserted replaced
56092:1ba075db8fe4 56093:4eeb73a1feec
   367   in one_line_proof ^ isar_proof end
   367   in one_line_proof ^ isar_proof end
   368 
   368 
   369 fun isar_proof_would_be_a_good_idea smt_proofs (meth, play) =
   369 fun isar_proof_would_be_a_good_idea smt_proofs (meth, play) =
   370   (case play of
   370   (case play of
   371     Played _ => meth = SMT2_Method andalso smt_proofs <> SOME true
   371     Played _ => meth = SMT2_Method andalso smt_proofs <> SOME true
   372   | Play_Timed_Out _ => true
   372   | Play_Timed_Out time => Time.> (time, Time.zeroTime)
   373   | Play_Failed => true
   373   | Play_Failed => true)
   374   | Not_Played => false)
       
   375 
   374 
   376 fun proof_text ctxt debug isar_proofs smt_proofs isar_params num_chained
   375 fun proof_text ctxt debug isar_proofs smt_proofs isar_params num_chained
   377     (one_line_params as (preplay, _, _, _, _, _)) =
   376     (one_line_params as (preplay, _, _, _, _, _)) =
   378   (if isar_proofs = SOME true orelse
   377   (if isar_proofs = SOME true orelse
   379       (isar_proofs = NONE andalso isar_proof_would_be_a_good_idea smt_proofs preplay) then
   378       (isar_proofs = NONE andalso isar_proof_would_be_a_good_idea smt_proofs preplay) then