src/HOL/Tools/try0.ML
changeset 74508 3315c551fe6e
parent 73386 3fb201ca8fb5
child 74870 d54b3c96ee50
--- a/src/HOL/Tools/try0.ML	Wed Oct 13 10:35:01 2021 +0200
+++ b/src/HOL/Tools/try0.ML	Wed Oct 13 11:04:35 2021 +0200
@@ -6,9 +6,7 @@
 
 signature TRY0 =
 sig
-  val try0N : string
   val noneN : string
-
   val silence_methods : bool -> Proof.context -> Proof.context
   val try0 : Time.time option -> string list * string list * string list * string list ->
     Proof.state -> bool
@@ -17,7 +15,6 @@
 structure Try0 : TRY0 =
 struct
 
-val try0N = "try0";
 val noneN = "none";
 
 datatype mode = Auto_Try | Try | Normal;
@@ -191,8 +188,9 @@
   Outer_Syntax.command \<^command_keyword>\<open>try0\<close> "try a combination of proof methods"
     (Scan.optional parse_attrs ([], [], [], []) #>> try0_trans);
 
-fun try_try0 auto = generic_try0 (if auto then Auto_Try else Try) NONE ([], [], [], []);
-
-val _ = Try.tool_setup (try0N, (30, \<^system_option>\<open>auto_methods\<close>, try_try0));
+val _ =
+  Try.tool_setup
+   {name = "try0", weight = 30, auto_option = \<^system_option>\<open>auto_methods\<close>,
+    body = fn auto => generic_try0 (if auto then Auto_Try else Try) NONE ([], [], [], [])};
 
 end;