src/HOL/SMT.thy
changeset 58072 a86c962de77f
parent 58061 3d060f43accb
child 58360 dee1fd1cc631
--- a/src/HOL/SMT.thy	Thu Aug 28 16:58:26 2014 +0200
+++ b/src/HOL/SMT.thy	Thu Aug 28 16:58:26 2014 +0200
@@ -127,7 +127,7 @@
   Scan.optional Attrib.thms [] >>
     (fn thms => fn ctxt =>
       METHOD (fn facts => HEADGOAL (SMT_Solver.smt_tac ctxt (thms @ facts))))
-*} "apply an SMT solver to the current goal (based on SMT-LIB 2)"
+*} "apply an SMT solver to the current goal"
 
 
 subsection {* Configuration *}