src/HOL/Library/Eval_Witness.thy
changeset 30510 4120fc59dd85
parent 29608 564ea783ace8
child 30549 d2d7874648bd
equal deleted inserted replaced
30509:e19d5b459a61 30510:4120fc59dd85
    82 
    82 
    83 fun eval_tac ws = CSUBGOAL (fn (ct, i) => rtac (eval_witness_oracle (ct, ws)) i)
    83 fun eval_tac ws = CSUBGOAL (fn (ct, i) => rtac (eval_witness_oracle (ct, ws)) i)
    84 
    84 
    85 in
    85 in
    86   Method.simple_args (Scan.repeat Args.name) (fn ws => fn _ =>
    86   Method.simple_args (Scan.repeat Args.name) (fn ws => fn _ =>
    87     Method.SIMPLE_METHOD' (eval_tac ws))
    87     SIMPLE_METHOD' (eval_tac ws))
    88 end
    88 end
    89 *} "Evaluation with ML witnesses"
    89 *} "Evaluation with ML witnesses"
    90 
    90 
    91 
    91 
    92 subsection {* Toy Examples *}
    92 subsection {* Toy Examples *}