author | wenzelm |
Sat, 11 Dec 2021 11:24:48 +0100 | |
changeset 74913 | c2a2be496f35 |
parent 74563 | 042041c0ebeb |
child 74887 | 56247fdb8bbb |
permissions | -rw-r--r-- |
5822
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
1 |
(* Title: Pure/Isar/args.ML |
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
2 |
Author: Markus Wenzel, TU Muenchen |
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
3 |
|
58011
bc6bced136e5
tuned signature -- moved type src to Token, without aliases;
wenzelm
parents:
57944
diff
changeset
|
4 |
Quasi-inner syntax based on outer tokens: concrete argument syntax of |
27811 | 5 |
attributes, methods etc. |
5822
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
6 |
*) |
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
7 |
|
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
8 |
signature ARGS = |
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
9 |
sig |
30513 | 10 |
val context: Proof.context context_parser |
11 |
val theory: theory context_parser |
|
61814
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
12 |
val symbolic: Token.T parser |
30513 | 13 |
val $$$ : string -> string parser |
14 |
val add: string parser |
|
15 |
val del: string parser |
|
16 |
val colon: string parser |
|
17 |
val query: string parser |
|
18 |
val bang: string parser |
|
19 |
val query_colon: string parser |
|
20 |
val bang_colon: string parser |
|
53168 | 21 |
val parens: 'a parser -> 'a parser |
22 |
val bracks: 'a parser -> 'a parser |
|
23 |
val mode: string -> bool parser |
|
30513 | 24 |
val maybe: 'a parser -> 'a option parser |
60577 | 25 |
val name_token: Token.T parser |
26 |
val name: string parser |
|
69349
7cef9e386ffe
more accurate positions for "name" (quoted string) and "embedded" (cartouche): refer to content without delimiters, which is e.g. relevant for systematic selection/renaming of scope groups;
wenzelm
parents:
63120
diff
changeset
|
27 |
val name_position: (string * Position.T) parser |
55111 | 28 |
val cartouche_inner_syntax: string parser |
59809 | 29 |
val cartouche_input: Input.source parser |
59857 | 30 |
val text_token: Token.T parser |
59809 | 31 |
val text_input: Input.source parser |
56500
90f17a04567d
proper Args.name vs. Args.text as documented (in contrast to adhoc union in 75aaee32893d, which had to cope with more limited Args.T);
wenzelm
parents:
56499
diff
changeset
|
32 |
val text: string parser |
30513 | 33 |
val binding: binding parser |
34 |
val alt_name: string parser |
|
35 |
val liberal_name: string parser |
|
36 |
val var: indexname parser |
|
58012 | 37 |
val internal_source: Token.src parser |
61814
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
38 |
val internal_name: Token.name_value parser |
30513 | 39 |
val internal_typ: typ parser |
40 |
val internal_term: term parser |
|
41 |
val internal_fact: thm list parser |
|
42 |
val internal_attribute: (morphism -> attribute) parser |
|
58017 | 43 |
val internal_declaration: declaration parser |
58012 | 44 |
val named_source: (Token.T -> Token.src) -> Token.src parser |
30513 | 45 |
val named_typ: (string -> typ) -> typ parser |
46 |
val named_term: (string -> term) -> term parser |
|
57942
e5bec882fdd0
more informative Token.Fact: retain name of dynamic fact (without selection);
wenzelm
parents:
56500
diff
changeset
|
47 |
val named_fact: (string -> string option * thm list) -> thm list parser |
58017 | 48 |
val named_attribute: (string * Position.T -> morphism -> attribute) -> |
49 |
(morphism -> attribute) parser |
|
59064 | 50 |
val text_declaration: (Input.source -> declaration) -> declaration parser |
59649 | 51 |
val cartouche_declaration: (Input.source -> declaration) -> declaration parser |
30513 | 52 |
val typ_abbrev: typ context_parser |
53 |
val typ: typ context_parser |
|
54 |
val term: term context_parser |
|
55155 | 55 |
val term_pattern: term context_parser |
30513 | 56 |
val term_abbrev: term context_parser |
57 |
val prop: term context_parser |
|
55951
c07d184aebe9
tuned signature -- more uniform check_type_name/read_type_name;
wenzelm
parents:
55915
diff
changeset
|
58 |
val type_name: {proper: bool, strict: bool} -> string context_parser |
55954 | 59 |
val const: {proper: bool, strict: bool} -> string context_parser |
30514 | 60 |
val goal_spec: ((int -> tactic) -> tactic) context_parser |
5822
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
61 |
end; |
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
62 |
|
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
63 |
structure Args: ARGS = |
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
64 |
struct |
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
65 |
|
27811 | 66 |
(** argument scanners **) |
5822
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
67 |
|
27371 | 68 |
(* context *) |
69 |
||
70 |
fun context x = (Scan.state >> Context.proof_of) x; |
|
71 |
fun theory x = (Scan.state >> Context.theory_of) x; |
|
72 |
||
73 |
||
27811 | 74 |
(* basic *) |
5878 | 75 |
|
56201 | 76 |
val ident = Parse.token |
36950 | 77 |
(Parse.short_ident || Parse.long_ident || Parse.sym_ident || Parse.term_var || |
78 |
Parse.type_ident || Parse.type_var || Parse.number); |
|
5878 | 79 |
|
56500
90f17a04567d
proper Args.name vs. Args.text as documented (in contrast to adhoc union in 75aaee32893d, which had to cope with more limited Args.T);
wenzelm
parents:
56499
diff
changeset
|
80 |
val string = Parse.token Parse.string; |
56499
7e0178c84994
allow text cartouches in regular outer syntax categories "text" and "altstring";
wenzelm
parents:
56333
diff
changeset
|
81 |
val alt_string = Parse.token (Parse.alt_string || Parse.cartouche); |
56201 | 82 |
val symbolic = Parse.token (Parse.keyword_with Token.ident_or_symbolic); |
27811 | 83 |
|
55914
c5b752d549e3
clarified init_assignable: make double-sure that initial values are reset;
wenzelm
parents:
55828
diff
changeset
|
84 |
fun $$$ x = |
56201 | 85 |
(ident || Parse.token Parse.keyword) :|-- (fn tok => |
56063 | 86 |
let val y = Token.content_of tok in |
87 |
if x = y |
|
56202 | 88 |
then (Token.assign (SOME (Token.Literal (false, Markup.quasi_keyword))) tok; Scan.succeed x) |
56063 | 89 |
else Scan.fail |
90 |
end); |
|
5878 | 91 |
|
10035 | 92 |
val add = $$$ "add"; |
93 |
val del = $$$ "del"; |
|
8803 | 94 |
val colon = $$$ ":"; |
10035 | 95 |
val query = $$$ "?"; |
96 |
val bang = $$$ "!"; |
|
20111 | 97 |
val query_colon = $$$ "?" ^^ $$$ ":"; |
98 |
val bang_colon = $$$ "!" ^^ $$$ ":"; |
|
10035 | 99 |
|
8803 | 100 |
fun parens scan = $$$ "(" |-- scan --| $$$ ")"; |
10150 | 101 |
fun bracks scan = $$$ "[" |-- scan --| $$$ "]"; |
53168 | 102 |
fun mode s = Scan.optional (parens ($$$ s) >> K true) false; |
15703 | 103 |
fun maybe scan = $$$ "_" >> K NONE || scan >> SOME; |
5878 | 104 |
|
60577 | 105 |
val name_token = ident || string; |
106 |
val name = name_token >> Token.content_of; |
|
69349
7cef9e386ffe
more accurate positions for "name" (quoted string) and "embedded" (cartouche): refer to content without delimiters, which is e.g. relevant for systematic selection/renaming of scope groups;
wenzelm
parents:
63120
diff
changeset
|
107 |
val name_position = name_token >> (Input.source_content o Token.input_of); |
60577 | 108 |
|
56201 | 109 |
val cartouche = Parse.token Parse.cartouche; |
55111 | 110 |
val cartouche_inner_syntax = cartouche >> Token.inner_syntax_of; |
59809 | 111 |
val cartouche_input = cartouche >> Token.input_of; |
55045
99056d23e05b
cartouche within nested args (attributes, methods, etc.);
wenzelm
parents:
55033
diff
changeset
|
112 |
|
74563 | 113 |
val text_token = Parse.token (Parse.embedded || Parse.verbatim); |
59809 | 114 |
val text_input = text_token >> Token.input_of; |
56500
90f17a04567d
proper Args.name vs. Args.text as documented (in contrast to adhoc union in 75aaee32893d, which had to cope with more limited Args.T);
wenzelm
parents:
56499
diff
changeset
|
115 |
val text = text_token >> Token.content_of; |
90f17a04567d
proper Args.name vs. Args.text as documented (in contrast to adhoc union in 75aaee32893d, which had to cope with more limited Args.T);
wenzelm
parents:
56499
diff
changeset
|
116 |
|
69349
7cef9e386ffe
more accurate positions for "name" (quoted string) and "embedded" (cartouche): refer to content without delimiters, which is e.g. relevant for systematic selection/renaming of scope groups;
wenzelm
parents:
63120
diff
changeset
|
117 |
val binding = Parse.input name >> (Binding.make o Input.source_content); |
36959
f5417836dbea
renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents:
36950
diff
changeset
|
118 |
val alt_name = alt_string >> Token.content_of; |
61814
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
119 |
val liberal_name = (symbolic >> Token.content_of) || name; |
8233 | 120 |
|
63120
629a4c5e953e
embedded content may be delimited via cartouches;
wenzelm
parents:
61814
diff
changeset
|
121 |
val var = |
629a4c5e953e
embedded content may be delimited via cartouches;
wenzelm
parents:
61814
diff
changeset
|
122 |
(ident >> Token.content_of) :|-- (fn x => |
629a4c5e953e
embedded content may be delimited via cartouches;
wenzelm
parents:
61814
diff
changeset
|
123 |
(case Lexicon.read_variable x of SOME v => Scan.succeed v | NONE => Scan.fail)); |
5878 | 124 |
|
5822
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
125 |
|
15703 | 126 |
(* values *) |
127 |
||
27811 | 128 |
fun value dest = Scan.some (fn arg => |
36959
f5417836dbea
renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents:
36950
diff
changeset
|
129 |
(case Token.get_value arg of SOME v => (SOME (dest v) handle Match => NONE) | NONE => NONE)); |
15703 | 130 |
|
58012 | 131 |
val internal_source = value (fn Token.Source src => src); |
61814
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
132 |
val internal_name = value (fn Token.Name (a, _) => a); |
36959
f5417836dbea
renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents:
36950
diff
changeset
|
133 |
val internal_typ = value (fn Token.Typ T => T); |
f5417836dbea
renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents:
36950
diff
changeset
|
134 |
val internal_term = value (fn Token.Term t => t); |
57942
e5bec882fdd0
more informative Token.Fact: retain name of dynamic fact (without selection);
wenzelm
parents:
56500
diff
changeset
|
135 |
val internal_fact = value (fn Token.Fact (_, ths) => ths); |
36959
f5417836dbea
renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents:
36950
diff
changeset
|
136 |
val internal_attribute = value (fn Token.Attribute att => att); |
58017 | 137 |
val internal_declaration = value (fn Token.Declaration decl => decl); |
15703 | 138 |
|
61814
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
139 |
fun named_source read = |
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
140 |
internal_source || name_token >> Token.evaluate Token.Source read; |
58012 | 141 |
|
60577 | 142 |
fun named_typ read = |
74563 | 143 |
internal_typ || |
144 |
Parse.token Parse.embedded >> Token.evaluate Token.Typ (read o Token.inner_syntax_of); |
|
60577 | 145 |
|
146 |
fun named_term read = |
|
74563 | 147 |
internal_term || |
148 |
Parse.token Parse.embedded >> Token.evaluate Token.Term (read o Token.inner_syntax_of); |
|
42464 | 149 |
|
57942
e5bec882fdd0
more informative Token.Fact: retain name of dynamic fact (without selection);
wenzelm
parents:
56500
diff
changeset
|
150 |
fun named_fact get = |
e5bec882fdd0
more informative Token.Fact: retain name of dynamic fact (without selection);
wenzelm
parents:
56500
diff
changeset
|
151 |
internal_fact || |
61814
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
152 |
name_token >> Token.evaluate Token.Fact (get o Token.content_of) >> #2 || |
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
153 |
alt_string >> Token.evaluate Token.Fact (get o Token.inner_syntax_of) >> #2; |
42464 | 154 |
|
36959
f5417836dbea
renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
wenzelm
parents:
36950
diff
changeset
|
155 |
fun named_attribute att = |
42464 | 156 |
internal_attribute || |
61814
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
157 |
name_token >> |
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
158 |
Token.evaluate Token.Attribute (fn tok => att (Token.content_of tok, Token.pos_of tok)); |
15703 | 159 |
|
58017 | 160 |
fun text_declaration read = |
61814
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
161 |
internal_declaration || text_token >> Token.evaluate Token.Declaration (read o Token.input_of); |
58017 | 162 |
|
59649 | 163 |
fun cartouche_declaration read = |
61814
1ca1142e1711
clarified type Token.src: plain token list, with usual implicit value assignment;
wenzelm
parents:
60577
diff
changeset
|
164 |
internal_declaration || cartouche >> Token.evaluate Token.Declaration (read o Token.input_of); |
59649 | 165 |
|
15703 | 166 |
|
5878 | 167 |
(* terms and types *) |
168 |
||
42360 | 169 |
val typ_abbrev = Scan.peek (named_typ o Proof_Context.read_typ_abbrev o Context.proof_of); |
25331 | 170 |
val typ = Scan.peek (named_typ o Syntax.read_typ o Context.proof_of); |
24508
c8b82fec6447
replaced ProofContext.read_term/prop by general Syntax.read_term/prop;
wenzelm
parents:
24244
diff
changeset
|
171 |
val term = Scan.peek (named_term o Syntax.read_term o Context.proof_of); |
55155 | 172 |
val term_pattern = Scan.peek (named_term o Proof_Context.read_term_pattern o Context.proof_of); |
42360 | 173 |
val term_abbrev = Scan.peek (named_term o Proof_Context.read_term_abbrev o Context.proof_of); |
24508
c8b82fec6447
replaced ProofContext.read_term/prop by general Syntax.read_term/prop;
wenzelm
parents:
24244
diff
changeset
|
174 |
val prop = Scan.peek (named_term o Syntax.read_prop o Context.proof_of); |
18635 | 175 |
|
5878 | 176 |
|
15703 | 177 |
(* type and constant names *) |
178 |
||
55951
c07d184aebe9
tuned signature -- more uniform check_type_name/read_type_name;
wenzelm
parents:
55915
diff
changeset
|
179 |
fun type_name flags = |
56002 | 180 |
Scan.peek (named_typ o Proof_Context.read_type_name flags o Context.proof_of) |
18998 | 181 |
>> (fn Type (c, _) => c | TFree (a, _) => a | _ => ""); |
15703 | 182 |
|
55954 | 183 |
fun const flags = |
56002 | 184 |
Scan.peek (named_term o Proof_Context.read_const flags o Context.proof_of) |
18998 | 185 |
>> (fn Const (c, _) => c | Free (x, _) => x | _ => ""); |
7553 | 186 |
|
15703 | 187 |
|
27811 | 188 |
(* improper method arguments *) |
15703 | 189 |
|
8536 | 190 |
val from_to = |
36950 | 191 |
Parse.nat -- ($$$ "-" |-- Parse.nat) >> (fn (i, j) => fn tac => Seq.INTERVAL tac i j) || |
192 |
Parse.nat --| $$$ "-" >> (fn i => fn tac => fn st => Seq.INTERVAL tac i (Thm.nprems_of st) st) || |
|
193 |
Parse.nat >> (fn i => fn tac => tac i) || |
|
15703 | 194 |
$$$ "!" >> K ALLGOALS; |
8536 | 195 |
|
56202 | 196 |
val goal = Parse.keyword_improper "[" |-- Parse.!!! (from_to --| Parse.keyword_improper "]"); |
30514 | 197 |
fun goal_spec x = Scan.lift (Scan.optional goal (fn tac => tac 1)) x; |
8233 | 198 |
|
5822
3f824514ad88
Concrete argument syntax (for attributes, methods etc.).
wenzelm
parents:
diff
changeset
|
199 |
end; |