src/HOL/ex/CASC_Setup.thy
changeset 43161 27dcda8fc89b
parent 42827 8bfdcaf30551
child 43205 23b81469499f
equal deleted inserted replaced
43160:d4f347508cd4 43161:27dcda8fc89b
    61    ORELSE
    61    ORELSE
    62    SOLVE_TIMEOUT max_secs "fastsimp" (ALLGOALS (fast_simp_tac ctxt))
    62    SOLVE_TIMEOUT max_secs "fastsimp" (ALLGOALS (fast_simp_tac ctxt))
    63 *}
    63 *}
    64 
    64 
    65 method_setup isabellep = {*
    65 method_setup isabellep = {*
    66   Scan.lift Parse.nat >>
    66   Scan.lift (Scan.optional Parse.nat 1) >>
    67     (fn m => fn ctxt => SIMPLE_METHOD (isabellep_tac ctxt m))
    67     (fn m => fn ctxt => SIMPLE_METHOD (isabellep_tac ctxt m))
    68 *} ""
    68 *} "combination of Isabelle provers and oracles for CASC"
    69 
    69 
    70 end
    70 end