3 Author: Amine Chaieb, TU Muenchen
6 header {* Generic reflection and reification *}
10 uses ("reflection.ML")
13 lemma ext2: "(\<forall>x. f x = g x) \<Longrightarrow> f = g"
18 method_setup reify = {*
20 Method.syntax (Attrib.thms --
21 Scan.option (Scan.lift (Args.$$$ "(") |-- Args.term --| Scan.lift (Args.$$$ ")"))) src #>
22 (fn ((eqs, to), ctxt) => Method.SIMPLE_METHOD' (Reflection.genreify_tac ctxt eqs to))
23 *} "partial automatic reification"
25 method_setup reflection = {*
27 Method.syntax (Attrib.thms --
28 Scan.option (Scan.lift (Args.$$$ "(") |-- Args.term --| Scan.lift (Args.$$$ ")"))) src #>
29 (fn ((ths, to), ctxt) => Method.SIMPLE_METHOD' (Reflection.reflection_tac ctxt ths to))
30 *} "reflection method"