src/HOL/Tools/try0.ML
changeset 52641 c56b6fa636e8
parent 52639 df830310e550
child 52643 34c29356930e
equal deleted inserted replaced
52640:38679321b251 52641:c56b6fa636e8
     9   val try0N : string
     9   val try0N : string
    10   val noneN : string
    10   val noneN : string
    11   val try0 :
    11   val try0 :
    12     Time.time option -> string list * string list * string list * string list
    12     Time.time option -> string list * string list * string list * string list
    13     -> Proof.state -> bool
    13     -> Proof.state -> bool
    14   val setup : theory -> theory
       
    15 end;
    14 end;
    16 
    15 
    17 structure Try0 : TRY0 =
    16 structure Try0 : TRY0 =
    18 struct
    17 struct
    19 
    18 
   191     (Scan.optional parse_attrs ([], [], [], []) #>> try0_trans)
   190     (Scan.optional parse_attrs ([], [], [], []) #>> try0_trans)
   192 
   191 
   193 fun try_try0 auto =
   192 fun try_try0 auto =
   194   do_try0 (if auto then Auto_Try else Try) NONE ([], [], [], [])
   193   do_try0 (if auto then Auto_Try else Try) NONE ([], [], [], [])
   195 
   194 
   196 val setup = Try.register_tool (try0N, (30, @{option auto_try0}, try_try0))
   195 val _ = Try.tool_setup (try0N, (30, @{option auto_try0}, try_try0))
   197 
   196 
   198 end;
   197 end;