src/HOL/Eisbach/Eisbach.thy
author wenzelm
Wed, 16 Dec 2015 16:31:36 +0100
changeset 61853 fb7756087101
parent 60623 be39fe6c5620
child 61918 0f9e0106c378
permissions -rw-r--r--
rule_attribute and declaration_attribute implicitly support abstract closure, but mixed_attribute implementations need to be aware of Thm.is_free_dummy;

(*  Title:      HOL/Eisbach/Eisbach.thy
    Author:     Daniel Matichuk, NICTA/UNSW

Main entry point for Eisbach proof method language.
*)

theory Eisbach
imports Main
keywords
  "method" :: thy_decl and
  "conclusion"
  "declares"
  "methods"
  "\<bar>" "\<Rightarrow>"
  "uses"
begin

ML_file "parse_tools.ML"
ML_file "method_closure.ML"
ML_file "eisbach_rule_insts.ML"
ML_file "match_method.ML"
ML_file "eisbach_antiquotations.ML"

method solves methods m = (m; fail)

end