src/HOL/Tools/SMT/smt_solver.ML
changeset 59621 291934bac95e
parent 58061 3d060f43accb
child 59632 5980e75a204e
equal deleted inserted replaced
59620:92d7d8e4f1bf 59621:291934bac95e
   205         if not (Config.get ctxt SMT_Config.oracle) andalso is_some replay0
   205         if not (Config.get ctxt SMT_Config.oracle) andalso is_some replay0
   206         then the replay0 outer_ctxt replay_data lines
   206         then the replay0 outer_ctxt replay_data lines
   207         else oracle ()
   207         else oracle ()
   208     | (result, _) => raise SMT_Failure.SMT (SMT_Failure.Counterexample (result = Sat)))
   208     | (result, _) => raise SMT_Failure.SMT (SMT_Failure.Counterexample (result = Sat)))
   209 
   209 
   210   val cfalse = Thm.cterm_of @{theory} @{prop False}
   210   val cfalse = Thm.global_cterm_of @{theory} @{prop False}
   211 in
   211 in
   212 
   212 
   213 fun add_solver ({name, class, avail, command, options, smt_options, default_max_relevant, outcome,
   213 fun add_solver ({name, class, avail, command, options, smt_options, default_max_relevant, outcome,
   214     parse_proof = parse_proof0, replay = replay0} : solver_config) =
   214     parse_proof = parse_proof0, replay = replay0} : solver_config) =
   215   let
   215   let