| author | wenzelm | 
| Fri, 16 Jan 2009 21:24:33 +0100 | |
| changeset 29520 | 7402322256b0 | 
| parent 29004 | a5a91f387791 | 
| child 29581 | b3b33e0298eb | 
| permissions | -rw-r--r-- | 
| 5823 | 1 | (* Title: Pure/Isar/attrib.ML | 
| 2 | Author: Markus Wenzel, TU Muenchen | |
| 3 | ||
| 18734 | 4 | Symbolic representation of attributes -- with name and syntax. | 
| 5823 | 5 | *) | 
| 6 | ||
| 7 | signature ATTRIB = | |
| 8 | sig | |
| 27729 | 9 | type src = Args.src | 
| 28965 | 10 | type binding = Binding.T * src list | 
| 11 | val empty_binding: binding | |
| 27729 | 12 | val print_attributes: theory -> unit | 
| 16458 | 13 | val intern: theory -> xstring -> string | 
| 14 | val intern_src: theory -> src -> src | |
| 21031 | 15 | val pretty_attribs: Proof.context -> src list -> Pretty.T list | 
| 26891 | 16 | val defined: theory -> string -> bool | 
| 18734 | 17 | val attribute: theory -> src -> attribute | 
| 18 | val attribute_i: theory -> src -> attribute | |
| 26336 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 19 | val eval_thms: Proof.context -> (Facts.ref * src list) list -> thm list | 
| 18905 | 20 |   val map_specs: ('a -> 'att) ->
 | 
| 21 |     (('c * 'a list) * 'd) list -> (('c * 'att list) * 'd) list
 | |
| 22 |   val map_facts: ('a -> 'att) ->
 | |
| 17105 
1b07a176a880
added map_specs/facts operators (from locale.ML);
 wenzelm parents: 
16934diff
changeset | 23 |     (('c * 'a list) * ('d * 'a list) list) list ->
 | 
| 18905 | 24 |     (('c * 'att list) * ('d * 'att list) list) list
 | 
| 20289 | 25 | val crude_closure: Proof.context -> src -> src | 
| 18734 | 26 | val add_attributes: (bstring * (src -> attribute) * string) list -> theory -> theory | 
| 25983 | 27 | val syntax: (Context.generic * Args.T list -> | 
| 28 | attribute * (Context.generic * Args.T list)) -> src -> attribute | |
| 29 | val no_args: attribute -> src -> attribute | |
| 30 | val add_del_args: attribute -> attribute -> src -> attribute | |
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 31 | val thm_sel: Args.T list -> Facts.interval list * Args.T list | 
| 25983 | 32 | val thm: Context.generic * Args.T list -> thm * (Context.generic * Args.T list) | 
| 33 | val thms: Context.generic * Args.T list -> thm list * (Context.generic * Args.T list) | |
| 34 | val multi_thm: Context.generic * Args.T list -> thm list * (Context.generic * Args.T list) | |
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 35 | val print_configs: Proof.context -> unit | 
| 25983 | 36 | val internal: (morphism -> attribute) -> src | 
| 24126 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 37 | val register_config: Config.value Config.T -> theory -> theory | 
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 38 | val config_bool: bstring -> bool -> bool Config.T * (theory -> theory) | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 39 | val config_int: bstring -> int -> int Config.T * (theory -> theory) | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 40 | val config_string: bstring -> string -> string Config.T * (theory -> theory) | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 41 | val config_bool_global: bstring -> bool -> bool Config.T * (theory -> theory) | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 42 | val config_int_global: bstring -> int -> int Config.T * (theory -> theory) | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 43 | val config_string_global: bstring -> string -> string Config.T * (theory -> theory) | 
| 5823 | 44 | end; | 
| 45 | ||
| 46 | structure Attrib: ATTRIB = | |
| 47 | struct | |
| 48 | ||
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 49 | structure T = OuterLex; | 
| 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 50 | structure P = OuterParse; | 
| 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 51 | |
| 28084 
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
 wenzelm parents: 
28083diff
changeset | 52 | |
| 
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
 wenzelm parents: 
28083diff
changeset | 53 | (* source and bindings *) | 
| 
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
 wenzelm parents: 
28083diff
changeset | 54 | |
| 15703 | 55 | type src = Args.src; | 
| 56 | ||
| 28965 | 57 | type binding = Binding.T * src list; | 
| 58 | val empty_binding: binding = (Binding.empty, []); | |
| 28084 
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
 wenzelm parents: 
28083diff
changeset | 59 | |
| 
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
 wenzelm parents: 
28083diff
changeset | 60 | |
| 27729 | 61 | |
| 18734 | 62 | (** named attributes **) | 
| 18636 | 63 | |
| 18734 | 64 | (* theory data *) | 
| 5823 | 65 | |
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 66 | structure Attributes = TheoryDataFun | 
| 22846 | 67 | ( | 
| 18734 | 68 | type T = (((src -> attribute) * string) * stamp) NameSpace.table; | 
| 16344 | 69 | val empty = NameSpace.empty_table; | 
| 6546 | 70 | val copy = I; | 
| 16458 | 71 | val extend = I; | 
| 23655 
d2d1138e0ddc
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
 wenzelm parents: 
23577diff
changeset | 72 | fun merge _ tables : T = NameSpace.merge_tables (eq_snd (op =)) tables handle Symtab.DUP dup => | 
| 
d2d1138e0ddc
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
 wenzelm parents: 
23577diff
changeset | 73 |     error ("Attempt to merge different versions of attribute " ^ quote dup);
 | 
| 22846 | 74 | ); | 
| 5823 | 75 | |
| 22846 | 76 | fun print_attributes thy = | 
| 77 | let | |
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 78 | val attribs = Attributes.get thy; | 
| 22846 | 79 | fun prt_attr (name, ((_, comment), _)) = Pretty.block | 
| 80 | [Pretty.str (name ^ ":"), Pretty.brk 2, Pretty.str comment]; | |
| 81 | in | |
| 82 | [Pretty.big_list "attributes:" (map prt_attr (NameSpace.extern_table attribs))] | |
| 83 | |> Pretty.chunks |> Pretty.writeln | |
| 84 | end; | |
| 7611 | 85 | |
| 5823 | 86 | |
| 21031 | 87 | (* name space *) | 
| 15703 | 88 | |
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 89 | val intern = NameSpace.intern o #1 o Attributes.get; | 
| 15703 | 90 | val intern_src = Args.map_name o intern; | 
| 91 | ||
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 92 | val extern = NameSpace.extern o #1 o Attributes.get o ProofContext.theory_of; | 
| 21031 | 93 | |
| 94 | ||
| 95 | (* pretty printing *) | |
| 96 | ||
| 97 | fun pretty_attribs _ [] = [] | |
| 98 | | pretty_attribs ctxt srcs = | |
| 99 | [Pretty.enclose "[" "]" | |
| 100 | (Pretty.commas (map (Args.pretty_src ctxt o Args.map_name (extern ctxt)) srcs))]; | |
| 101 | ||
| 15703 | 102 | |
| 18734 | 103 | (* get attributes *) | 
| 5823 | 104 | |
| 26891 | 105 | val defined = Symtab.defined o #2 o Attributes.get; | 
| 106 | ||
| 18734 | 107 | fun attribute_i thy = | 
| 5823 | 108 | let | 
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 109 | val attrs = #2 (Attributes.get thy); | 
| 5879 | 110 | fun attr src = | 
| 16344 | 111 | let val ((name, _), pos) = Args.dest_src src in | 
| 17412 | 112 | (case Symtab.lookup attrs name of | 
| 15531 | 113 |           NONE => error ("Unknown attribute: " ^ quote name ^ Position.str_of pos)
 | 
| 27751 | 114 | | SOME ((att, _), _) => (Position.report (Markup.attribute name) pos; att src)) | 
| 5823 | 115 | end; | 
| 116 | in attr end; | |
| 117 | ||
| 18734 | 118 | fun attribute thy = attribute_i thy o intern_src thy; | 
| 18636 | 119 | |
| 24723 | 120 | fun eval_thms ctxt args = ProofContext.note_thmss Thm.theoremK | 
| 28965 | 121 | [((Binding.empty, []), | 
| 28083 
103d9282a946
explicit type Name.binding for higher-specification elements;
 wenzelm parents: 
27865diff
changeset | 122 | map (apsnd (map (attribute (ProofContext.theory_of ctxt)))) args)] ctxt | 
| 26685 | 123 | |> fst |> maps snd; | 
| 24723 | 124 | |
| 5823 | 125 | |
| 17105 
1b07a176a880
added map_specs/facts operators (from locale.ML);
 wenzelm parents: 
16934diff
changeset | 126 | (* attributed declarations *) | 
| 
1b07a176a880
added map_specs/facts operators (from locale.ML);
 wenzelm parents: 
16934diff
changeset | 127 | |
| 
1b07a176a880
added map_specs/facts operators (from locale.ML);
 wenzelm parents: 
16934diff
changeset | 128 | fun map_specs f = map (apfst (apsnd (map f))); | 
| 
1b07a176a880
added map_specs/facts operators (from locale.ML);
 wenzelm parents: 
16934diff
changeset | 129 | fun map_facts f = map (apfst (apsnd (map f)) o apsnd (map (apsnd (map f)))); | 
| 
1b07a176a880
added map_specs/facts operators (from locale.ML);
 wenzelm parents: 
16934diff
changeset | 130 | |
| 
1b07a176a880
added map_specs/facts operators (from locale.ML);
 wenzelm parents: 
16934diff
changeset | 131 | |
| 15703 | 132 | (* crude_closure *) | 
| 133 | ||
| 134 | (*Produce closure without knowing facts in advance! The following | |
| 18734 | 135 | works reasonably well for attribute parsers that do not peek at the | 
| 136 | thm structure.*) | |
| 15703 | 137 | |
| 138 | fun crude_closure ctxt src = | |
| 18734 | 139 | (try (fn () => attribute_i (ProofContext.theory_of ctxt) src | 
| 140 | (Context.Proof ctxt, Drule.asm_rl)) (); | |
| 15703 | 141 | Args.closure src); | 
| 142 | ||
| 143 | ||
| 5823 | 144 | (* add_attributes *) | 
| 145 | ||
| 146 | fun add_attributes raw_attrs thy = | |
| 147 | let | |
| 18734 | 148 | val new_attrs = | 
| 29004 | 149 | raw_attrs |> map (fn (name, att, comment) => (Binding.name name, ((att, comment), stamp ()))); | 
| 150 | fun add attrs = fold (snd oo NameSpace.bind (Sign.naming_of thy)) new_attrs attrs | |
| 23655 
d2d1138e0ddc
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
 wenzelm parents: 
23577diff
changeset | 151 |       handle Symtab.DUP dup => error ("Duplicate declaration of attributes " ^ quote dup);
 | 
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 152 | in Attributes.map add thy end; | 
| 5823 | 153 | |
| 5879 | 154 | |
| 25983 | 155 | (* attribute syntax *) | 
| 5879 | 156 | |
| 25983 | 157 | fun syntax scan src (st, th) = | 
| 158 | let val (f: attribute, st') = Args.syntax "attribute" scan src st | |
| 159 | in f (st', th) end; | |
| 5823 | 160 | |
| 25983 | 161 | fun no_args x = syntax (Scan.succeed x); | 
| 162 | ||
| 163 | fun add_del_args add del = syntax | |
| 164 | (Scan.lift (Args.add >> K add || Args.del >> K del || Scan.succeed add)); | |
| 5879 | 165 | |
| 166 | ||
| 25983 | 167 | |
| 168 | (** parsing attributed theorems **) | |
| 5879 | 169 | |
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 170 | val thm_sel = P.$$$ "(" |-- P.list1
 | 
| 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 171 | (P.nat --| P.minus -- P.nat >> Facts.FromTo || | 
| 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 172 | P.nat --| P.minus >> Facts.From || | 
| 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 173 | P.nat >> Facts.Single) --| P.$$$ ")"; | 
| 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 174 | |
| 18636 | 175 | local | 
| 176 | ||
| 21698 
43a842769765
thms etc.: proper treatment of internal_fact with selection;
 wenzelm parents: 
21658diff
changeset | 177 | val fact_name = Args.internal_fact >> K "<fact>" || Args.name; | 
| 
43a842769765
thms etc.: proper treatment of internal_fact with selection;
 wenzelm parents: 
21658diff
changeset | 178 | |
| 26336 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 179 | fun gen_thm pick = Scan.depend (fn context => | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 180 | let | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 181 | val thy = Context.theory_of context; | 
| 26685 | 182 | val get = Context.cases (PureThy.get_fact context) ProofContext.get_fact context; | 
| 26361 | 183 | val get_fact = get o Facts.Fact; | 
| 27820 | 184 | fun get_named pos name = get (Facts.Named ((name, pos), NONE)); | 
| 26336 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 185 | in | 
| 27820 | 186 | P.$$$ "[" |-- Args.attribs (intern thy) --| P.$$$ "]" >> (fn srcs => | 
| 24008 | 187 | let | 
| 26336 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 188 | val atts = map (attribute_i thy) srcs; | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 189 | val (context', th') = Library.apply atts (context, Drule.dummy_thm); | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 190 | in (context', pick "" [th']) end) | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 191 | || | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 192 | (Scan.ahead Args.alt_name -- Args.named_fact get_fact | 
| 27820 | 193 |       >> (fn (s, fact) => ("", Facts.Fact s, fact)) ||
 | 
| 194 | Scan.ahead (P.position fact_name) :|-- (fn (name, pos) => | |
| 195 | Args.named_fact (get_named pos) -- Scan.option thm_sel | |
| 196 | >> (fn (fact, sel) => (name, Facts.Named ((name, pos), sel), fact)))) | |
| 26336 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 197 | -- Args.opt_attribs (intern thy) >> (fn ((name, thmref, fact), srcs) => | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 198 | let | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 199 | val ths = Facts.select thmref fact; | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 200 | val atts = map (attribute_i thy) srcs; | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 201 | val (context', ths') = foldl_map (Library.apply atts) (context, ths); | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 202 | in (context', pick name ths') end) | 
| 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 203 | end); | 
| 15456 
956d6acacf89
Specific theorems in a named list of theorems can now be referred to
 berghofe parents: 
15117diff
changeset | 204 | |
| 18636 | 205 | in | 
| 206 | ||
| 26336 
a0e2b706ce73
renamed datatype thmref to Facts.ref, tuned interfaces;
 wenzelm parents: 
25983diff
changeset | 207 | val thm = gen_thm Facts.the_single; | 
| 18998 | 208 | val multi_thm = gen_thm (K I); | 
| 19482 
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
 wenzelm parents: 
19473diff
changeset | 209 | val thms = Scan.repeat multi_thm >> flat; | 
| 18636 | 210 | |
| 211 | end; | |
| 212 | ||
| 5823 | 213 | |
| 5879 | 214 | |
| 25983 | 215 | (** basic attributes **) | 
| 216 | ||
| 217 | (* internal *) | |
| 218 | ||
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 219 | fun internal att = Args.src (("Pure.attribute", [T.mk_attribute att]), Position.none);
 | 
| 25983 | 220 | |
| 221 | val internal_att = | |
| 222 | syntax (Scan.lift Args.internal_attribute >> Morphism.form); | |
| 223 | ||
| 224 | ||
| 225 | (* tags *) | |
| 226 | ||
| 27865 
27a8ad9612a3
moved basic thm operations from structure PureThy to Thm (cf. more_thm.ML);
 wenzelm parents: 
27820diff
changeset | 227 | val tagged = syntax (Scan.lift (Args.name -- Args.name) >> Thm.tag); | 
| 
27a8ad9612a3
moved basic thm operations from structure PureThy to Thm (cf. more_thm.ML);
 wenzelm parents: 
27820diff
changeset | 228 | val untagged = syntax (Scan.lift Args.name >> Thm.untag); | 
| 25983 | 229 | |
| 27865 
27a8ad9612a3
moved basic thm operations from structure PureThy to Thm (cf. more_thm.ML);
 wenzelm parents: 
27820diff
changeset | 230 | val kind = syntax (Scan.lift Args.name >> Thm.kind); | 
| 25983 | 231 | |
| 232 | ||
| 233 | (* rule composition *) | |
| 234 | ||
| 235 | val COMP_att = | |
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 236 | syntax (Scan.lift (Scan.optional (Args.bracks P.nat) 1) -- thm | 
| 25983 | 237 | >> (fn (i, B) => Thm.rule_attribute (fn _ => fn A => Drule.compose_single (A, i, B)))); | 
| 238 | ||
| 239 | val THEN_att = | |
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 240 | syntax (Scan.lift (Scan.optional (Args.bracks P.nat) 1) -- thm | 
| 25983 | 241 | >> (fn (i, B) => Thm.rule_attribute (fn _ => fn A => A RSN (i, B)))); | 
| 242 | ||
| 243 | val OF_att = | |
| 244 | syntax (thms >> (fn Bs => Thm.rule_attribute (fn _ => fn A => Bs MRS A))); | |
| 245 | ||
| 246 | ||
| 247 | (* rename_abs *) | |
| 248 | ||
| 249 | val rename_abs = syntax | |
| 250 | (Scan.lift (Scan.repeat (Args.maybe Args.name) >> (apsnd o Drule.rename_bvars'))); | |
| 251 | ||
| 252 | ||
| 253 | (* unfold / fold definitions *) | |
| 254 | ||
| 255 | fun unfolded_syntax rule = | |
| 256 | syntax (thms >> | |
| 257 | (fn ths => Thm.rule_attribute (fn context => rule (Context.proof_of context) ths))); | |
| 258 | ||
| 259 | val unfolded = unfolded_syntax LocalDefs.unfold; | |
| 260 | val folded = unfolded_syntax LocalDefs.fold; | |
| 261 | ||
| 262 | ||
| 263 | (* rule cases *) | |
| 5823 | 264 | |
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 265 | val consumes = syntax (Scan.lift (Scan.optional P.nat 1) >> RuleCases.consumes); | 
| 25983 | 266 | val case_names = syntax (Scan.lift (Scan.repeat1 Args.name) >> RuleCases.case_names); | 
| 267 | val case_conclusion = | |
| 268 | syntax (Scan.lift (Args.name -- Scan.repeat Args.name) >> RuleCases.case_conclusion); | |
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 269 | val params = syntax (Scan.lift (P.and_list1 (Scan.repeat Args.name)) >> RuleCases.params); | 
| 25983 | 270 | |
| 271 | ||
| 272 | (* rule format *) | |
| 273 | ||
| 274 | val rule_format = syntax (Args.mode "no_asm" | |
| 275 | >> (fn true => ObjectLogic.rule_format_no_asm | false => ObjectLogic.rule_format)); | |
| 276 | ||
| 277 | val elim_format = no_args (Thm.rule_attribute (K Tactic.make_elim)); | |
| 278 | ||
| 279 | ||
| 280 | (* misc rules *) | |
| 281 | ||
| 282 | val standard = no_args (Thm.rule_attribute (K Drule.standard)); | |
| 283 | ||
| 26715 
00ff79ab6e6b
no_vars: reset body mode, i.e. invent global frees (which are acceptable to Variable.auto_fixes);
 wenzelm parents: 
26685diff
changeset | 284 | val no_vars = no_args (Thm.rule_attribute (fn context => fn th => | 
| 
00ff79ab6e6b
no_vars: reset body mode, i.e. invent global frees (which are acceptable to Variable.auto_fixes);
 wenzelm parents: 
26685diff
changeset | 285 | let | 
| 
00ff79ab6e6b
no_vars: reset body mode, i.e. invent global frees (which are acceptable to Variable.auto_fixes);
 wenzelm parents: 
26685diff
changeset | 286 | val ctxt = Variable.set_body false (Context.proof_of context); | 
| 
00ff79ab6e6b
no_vars: reset body mode, i.e. invent global frees (which are acceptable to Variable.auto_fixes);
 wenzelm parents: 
26685diff
changeset | 287 | val ((_, [th']), _) = Variable.import_thms true [th] ctxt; | 
| 25983 | 288 | in th' end)); | 
| 289 | ||
| 290 | val eta_long = | |
| 291 | no_args (Thm.rule_attribute (K (Conv.fconv_rule Drule.eta_long_conversion))); | |
| 292 | ||
| 293 | val rotated = syntax | |
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 294 | (Scan.lift (Scan.optional P.int 1) >> (fn n => Thm.rule_attribute (K (rotate_prems n)))); | 
| 5879 | 295 | |
| 25983 | 296 | |
| 297 | (* theory setup *) | |
| 5823 | 298 | |
| 26463 | 299 | val _ = Context.>> (Context.map_theory | 
| 25983 | 300 | (add_attributes | 
| 301 |    [("attribute", internal_att, "internal attribute"),
 | |
| 302 |     ("tagged", tagged, "tagged theorem"),
 | |
| 303 |     ("untagged", untagged, "untagged theorem"),
 | |
| 304 |     ("kind", kind, "theorem kind"),
 | |
| 305 |     ("COMP", COMP_att, "direct composition with rules (no lifting)"),
 | |
| 306 |     ("THEN", THEN_att, "resolution with rule"),
 | |
| 307 |     ("OF", OF_att, "rule applied to facts"),
 | |
| 308 |     ("rename_abs", rename_abs, "rename bound variables in abstractions"),
 | |
| 309 |     ("unfolded", unfolded, "unfolded definitions"),
 | |
| 310 |     ("folded", folded, "folded definitions"),
 | |
| 311 |     ("standard", standard, "result put into standard form"),
 | |
| 312 |     ("elim_format", elim_format, "destruct rule turned into elimination rule format"),
 | |
| 313 |     ("no_vars", no_vars, "frozen schematic vars"),
 | |
| 314 |     ("eta_long", eta_long, "put theorem into eta long beta normal form"),
 | |
| 315 |     ("consumes", consumes, "number of consumed facts"),
 | |
| 316 |     ("case_names", case_names, "named rule cases"),
 | |
| 317 |     ("case_conclusion", case_conclusion, "named conclusion of rule cases"),
 | |
| 318 |     ("params", params, "named rule parameters"),
 | |
| 319 |     ("atomize", no_args ObjectLogic.declare_atomize, "declaration of atomize rule"),
 | |
| 320 |     ("rulify", no_args ObjectLogic.declare_rulify, "declaration of rulify rule"),
 | |
| 321 |     ("rule_format", rule_format, "result put into standard rule format"),
 | |
| 322 |     ("rotated", rotated, "rotated theorem premises"),
 | |
| 323 |     ("defn", add_del_args LocalDefs.defn_add LocalDefs.defn_del,
 | |
| 26463 | 324 | "declaration of definitional transformations")])); | 
| 8633 | 325 | |
| 5823 | 326 | |
| 327 | ||
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 328 | (** configuration options **) | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 329 | |
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 330 | (* naming *) | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 331 | |
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 332 | structure Configs = TheoryDataFun | 
| 24713 | 333 | ( | 
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 334 | type T = Config.value Config.T Symtab.table; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 335 | val empty = Symtab.empty; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 336 | val copy = I; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 337 | val extend = I; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 338 | fun merge _ = Symtab.merge (K true); | 
| 24713 | 339 | ); | 
| 5823 | 340 | |
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 341 | fun print_configs ctxt = | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 342 | let | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 343 | val thy = ProofContext.theory_of ctxt; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 344 | fun prt (name, config) = | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 345 | let val value = Config.get ctxt config in | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 346 | Pretty.block [Pretty.str (name ^ ": " ^ Config.print_type value ^ " ="), Pretty.brk 1, | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 347 | Pretty.str (Config.print_value value)] | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 348 | end; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 349 | val configs = NameSpace.extern_table (#1 (Attributes.get thy), Configs.get thy); | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 350 | in Pretty.writeln (Pretty.big_list "configuration options" (map prt configs)) end; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 351 | |
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 352 | |
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 353 | (* concrete syntax *) | 
| 23988 
aa46577f4f44
added attribute "option" for setting configuration options;
 wenzelm parents: 
23937diff
changeset | 354 | |
| 24003 
da76d7e6435c
attribute "option": more elaborate syntax (with value parsing);
 wenzelm parents: 
23988diff
changeset | 355 | local | 
| 
da76d7e6435c
attribute "option": more elaborate syntax (with value parsing);
 wenzelm parents: 
23988diff
changeset | 356 | |
| 27820 | 357 | val equals = P.$$$ "="; | 
| 24003 
da76d7e6435c
attribute "option": more elaborate syntax (with value parsing);
 wenzelm parents: 
23988diff
changeset | 358 | |
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 359 | fun scan_value (Config.Bool _) = | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 360 | equals -- Args.$$$ "false" >> K (Config.Bool false) || | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 361 | equals -- Args.$$$ "true" >> K (Config.Bool true) || | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 362 | Scan.succeed (Config.Bool true) | 
| 27812 
af8edf3ab68c
unified Args.T with OuterLex.token, renamed some operations;
 wenzelm parents: 
27751diff
changeset | 363 | | scan_value (Config.Int _) = equals |-- P.int >> Config.Int | 
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 364 | | scan_value (Config.String _) = equals |-- Args.name >> Config.String; | 
| 24003 
da76d7e6435c
attribute "option": more elaborate syntax (with value parsing);
 wenzelm parents: 
23988diff
changeset | 365 | |
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 366 | fun scan_config thy config = | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 367 | let val config_type = Config.get_thy thy config | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 368 | in scan_value config_type >> (K o Thm.declaration_attribute o K o Config.put_generic config) end; | 
| 24003 
da76d7e6435c
attribute "option": more elaborate syntax (with value parsing);
 wenzelm parents: 
23988diff
changeset | 369 | |
| 
da76d7e6435c
attribute "option": more elaborate syntax (with value parsing);
 wenzelm parents: 
23988diff
changeset | 370 | in | 
| 
da76d7e6435c
attribute "option": more elaborate syntax (with value parsing);
 wenzelm parents: 
23988diff
changeset | 371 | |
| 24126 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 372 | fun register_config config thy = | 
| 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 373 | let | 
| 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 374 | val bname = Config.name_of config; | 
| 28965 | 375 | val name = Sign.full_bname thy bname; | 
| 24126 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 376 | in | 
| 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 377 | thy | 
| 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 378 | |> add_attributes [(bname, syntax (Scan.lift (scan_config thy config) >> Morphism.form), | 
| 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 379 | "configuration option")] | 
| 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 380 | |> Configs.map (Symtab.update (name, config)) | 
| 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 381 | end; | 
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 382 | |
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 383 | fun declare_config make coerce global name default = | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 384 | let | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 385 | val config_value = Config.declare global name (make default); | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 386 | val config = coerce config_value; | 
| 24126 
913e1fa904fb
turned simp_depth_limit into configuration option;
 wenzelm parents: 
24110diff
changeset | 387 | in (config, register_config config_value) end; | 
| 24110 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 388 | |
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 389 | val config_bool = declare_config Config.Bool Config.bool false; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 390 | val config_int = declare_config Config.Int Config.int false; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 391 | val config_string = declare_config Config.String Config.string false; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 392 | |
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 393 | val config_bool_global = declare_config Config.Bool Config.bool true; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 394 | val config_int_global = declare_config Config.Int Config.int true; | 
| 
4ab3084e311c
tuned config options: eliminated separate attribute "option";
 wenzelm parents: 
24030diff
changeset | 395 | val config_string_global = declare_config Config.String Config.string true; | 
| 24003 
da76d7e6435c
attribute "option": more elaborate syntax (with value parsing);
 wenzelm parents: 
23988diff
changeset | 396 | |
| 
da76d7e6435c
attribute "option": more elaborate syntax (with value parsing);
 wenzelm parents: 
23988diff
changeset | 397 | end; | 
| 23988 
aa46577f4f44
added attribute "option" for setting configuration options;
 wenzelm parents: 
23937diff
changeset | 398 | |
| 
aa46577f4f44
added attribute "option" for setting configuration options;
 wenzelm parents: 
23937diff
changeset | 399 | |
| 18636 | 400 | (* theory setup *) | 
| 5823 | 401 | |
| 26463 | 402 | val _ = Context.>> (Context.map_theory | 
| 24178 
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
 wenzelm parents: 
24126diff
changeset | 403 | (register_config Unify.trace_bound_value #> | 
| 
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
 wenzelm parents: 
24126diff
changeset | 404 | register_config Unify.search_bound_value #> | 
| 
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
 wenzelm parents: 
24126diff
changeset | 405 | register_config Unify.trace_simp_value #> | 
| 
4ff1dc2aa18d
turned Unify flags into configuration options (global only);
 wenzelm parents: 
24126diff
changeset | 406 | register_config Unify.trace_types_value #> | 
| 26463 | 407 | register_config MetaSimplifier.simp_depth_limit_value)); | 
| 5823 | 408 | |
| 409 | end; |