src/HOL/SMT.thy
changeset 58072 a86c962de77f
parent 58061 3d060f43accb
child 58360 dee1fd1cc631
equal deleted inserted replaced
58071:62ec5b1d2f2f 58072:a86c962de77f
   125 
   125 
   126 method_setup smt = {*
   126 method_setup smt = {*
   127   Scan.optional Attrib.thms [] >>
   127   Scan.optional Attrib.thms [] >>
   128     (fn thms => fn ctxt =>
   128     (fn thms => fn ctxt =>
   129       METHOD (fn facts => HEADGOAL (SMT_Solver.smt_tac ctxt (thms @ facts))))
   129       METHOD (fn facts => HEADGOAL (SMT_Solver.smt_tac ctxt (thms @ facts))))
   130 *} "apply an SMT solver to the current goal (based on SMT-LIB 2)"
   130 *} "apply an SMT solver to the current goal"
   131 
   131 
   132 
   132 
   133 subsection {* Configuration *}
   133 subsection {* Configuration *}
   134 
   134 
   135 text {*
   135 text {*