src/HOL/Tools/SMT/smt_solver.ML
changeset 42616 92715b528e78
parent 42320 1f09e4c680fc
child 46464 4cf5a84e2c05
equal deleted inserted replaced
42607:c8673078f915 42616:92715b528e78
   348       SMT_Failure.SMT (fail as SMT_Failure.Counterexample _) =>
   348       SMT_Failure.SMT (fail as SMT_Failure.Counterexample _) =>
   349         (SMT_Config.verbose_msg ctxt (str_of ctxt) fail; NONE)
   349         (SMT_Config.verbose_msg ctxt (str_of ctxt) fail; NONE)
   350     | SMT_Failure.SMT (fail as SMT_Failure.Time_Out) =>
   350     | SMT_Failure.SMT (fail as SMT_Failure.Time_Out) =>
   351         error ("SMT: Solver " ^ quote (SMT_Config.solver_of ctxt) ^ ": " ^
   351         error ("SMT: Solver " ^ quote (SMT_Config.solver_of ctxt) ^ ": " ^
   352           SMT_Failure.string_of_failure ctxt fail ^ " (setting the " ^
   352           SMT_Failure.string_of_failure ctxt fail ^ " (setting the " ^
   353           "configuration option " ^ SMT_Config.timeoutN ^ " might help)")
   353           "configuration option " ^ quote (Config.name_of SMT_Config.timeout) ^ " might help)")
   354     | SMT_Failure.SMT fail => error (str_of ctxt fail)
   354     | SMT_Failure.SMT fail => error (str_of ctxt fail)
   355 
   355 
   356   fun tag_rules thms = map_index (apsnd (pair NONE)) thms
   356   fun tag_rules thms = map_index (apsnd (pair NONE)) thms
   357   fun tag_prems thms = map (pair ~1 o pair NONE) thms
   357   fun tag_prems thms = map (pair ~1 o pair NONE) thms
   358 
   358