src/Pure/Pure.thy
changeset 63043 df83a961d3a8
parent 63039 1a20fd9cf281
child 63059 3f577308551e
--- a/src/Pure/Pure.thy	Mon Apr 25 17:37:36 2016 +0200
+++ b/src/Pure/Pure.thy	Mon Apr 25 19:41:39 2016 +0200
@@ -749,7 +749,8 @@
       (Parse_Spec.opt_thm_name ":" --
         ((Parse.binding -- Parse.opt_mixfix) --
           ((@{keyword "\<equiv>"} || @{keyword "=="}) |-- Parse.!!! Parse.termp)))
-    >> (Toplevel.proof o Proof.def_cmd));
+    >> (fn args => Toplevel.proof (fn state =>
+        (legacy_feature "Old 'def' command -- use 'define' instead"; Proof.def_cmd args state))));
 
 val _ =
   Outer_Syntax.command @{command_keyword consider} "state cases rule"