src/HOL/Tools/try0.ML
changeset 52641 c56b6fa636e8
parent 52639 df830310e550
child 52643 34c29356930e
--- a/src/HOL/Tools/try0.ML	Sat Jul 13 00:24:05 2013 +0200
+++ b/src/HOL/Tools/try0.ML	Sat Jul 13 00:50:49 2013 +0200
@@ -11,7 +11,6 @@
   val try0 :
     Time.time option -> string list * string list * string list * string list
     -> Proof.state -> bool
-  val setup : theory -> theory
 end;
 
 structure Try0 : TRY0 =
@@ -193,6 +192,6 @@
 fun try_try0 auto =
   do_try0 (if auto then Auto_Try else Try) NONE ([], [], [], [])
 
-val setup = Try.register_tool (try0N, (30, @{option auto_try0}, try_try0))
+val _ = Try.tool_setup (try0N, (30, @{option auto_try0}, try_try0))
 
 end;