ProgTutorial/Recipes/Timing.thy
changeset 239 b63c72776f03
parent 191 0150cf5982ae
child 346 0fea8b7a14a1
equal deleted inserted replaced
238:29787dcf7b2e 239:b63c72776f03
    31 let 
    31 let 
    32   val t_start = start_timing ();
    32   val t_start = start_timing ();
    33   val res = tac st;
    33   val res = tac st;
    34   val t_end = end_timing t_start;
    34   val t_end = end_timing t_start;
    35 in
    35 in
    36   (warning (#message t_end); res)
    36   (writeln (#message t_end); res)
    37 end*}
    37 end*}
    38 
    38 
    39 text {*
    39 text {*
    40   Note that this function, in addition to a tactic, also takes a state @{text
    40   Note that this function, in addition to a tactic, also takes a state @{text
    41   "st"} as argument and applies this state to the tactic (Line 4). The reason is that
    41   "st"} as argument and applies this state to the tactic (Line 4). The reason is that