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