more official legacy status;
authorwenzelm
Fri, 07 Oct 2016 10:46:34 +0200
changeset 64078 0b22328a353c
parent 64073 cffd5f537206
child 64079 ff26032b7f2a
more official legacy status;
src/HOL/Library/Old_SMT.thy
--- a/src/HOL/Library/Old_SMT.thy	Fri Oct 07 10:31:34 2016 +0200
+++ b/src/HOL/Library/Old_SMT.thy	Fri Oct 07 10:46:34 2016 +0200
@@ -142,7 +142,8 @@
 method_setup old_smt = \<open>
   Scan.optional Attrib.thms [] >>
     (fn thms => fn ctxt =>
-      METHOD (fn facts => HEADGOAL (Old_SMT_Solver.smt_tac ctxt (thms @ facts))))
+      (legacy_feature "Proof method \"old_smt\" will be discontinued soon -- use \"smt\" instead";
+       METHOD (fn facts => HEADGOAL (Old_SMT_Solver.smt_tac ctxt (thms @ facts)))))
 \<close> "apply an SMT solver to the current goal"