author | wenzelm |
Wed, 25 Sep 2024 10:38:46 +0200 | |
changeset 80950 | b4a6bee4621a |
parent 80882 | 2cdb00f797b1 |
child 80952 | a61ed25ba155 |
permissions | -rw-r--r-- |
42243 | 1 |
(* Title: Pure/Syntax/syntax_phases.ML |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
2 |
Author: Makarius |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
3 |
|
42243 | 4 |
Main phases of inner syntax processing, with standard implementations |
5 |
of parse/unparse operations. |
|
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
6 |
*) |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
7 |
|
42243 | 8 |
signature SYNTAX_PHASES = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
9 |
sig |
74571 | 10 |
val markup_free: Proof.context -> string -> Markup.T list |
63395 | 11 |
val reports_of_scope: Position.T list -> Position.report list |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
12 |
val decode_sort: term -> sort |
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
13 |
val decode_typ: term -> typ |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
14 |
val decode_term: Proof.context -> |
55922
710bc66f432c
more markup for inner syntax class/type names (notably for completion);
wenzelm
parents:
55829
diff
changeset
|
15 |
Position.report_text list * term Exn.result -> Position.report_text list * term Exn.result |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
16 |
val parse_ast_pattern: Proof.context -> string * string -> Ast.ast |
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
17 |
val term_of_typ: Proof.context -> typ -> term |
45429 | 18 |
val print_checks: Proof.context -> unit |
19 |
val typ_check: int -> string -> (Proof.context -> typ list -> typ list) -> |
|
20 |
Context.generic -> Context.generic |
|
21 |
val term_check: int -> string -> (Proof.context -> term list -> term list) -> |
|
22 |
Context.generic -> Context.generic |
|
23 |
val typ_uncheck: int -> string -> (Proof.context -> typ list -> typ list) -> |
|
24 |
Context.generic -> Context.generic |
|
25 |
val term_uncheck: int -> string -> (Proof.context -> term list -> term list) -> |
|
26 |
Context.generic -> Context.generic |
|
45444 | 27 |
val typ_check': int -> string -> |
28 |
(typ list -> Proof.context -> (typ list * Proof.context) option) -> |
|
29 |
Context.generic -> Context.generic |
|
30 |
val term_check': int -> string -> |
|
31 |
(term list -> Proof.context -> (term list * Proof.context) option) -> |
|
32 |
Context.generic -> Context.generic |
|
33 |
val typ_uncheck': int -> string -> |
|
34 |
(typ list -> Proof.context -> (typ list * Proof.context) option) -> |
|
35 |
Context.generic -> Context.generic |
|
36 |
val term_uncheck': int -> string -> |
|
37 |
(term list -> Proof.context -> (term list * Proof.context) option) -> |
|
38 |
Context.generic -> Context.generic |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
39 |
end |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
40 |
|
42243 | 41 |
structure Syntax_Phases: SYNTAX_PHASES = |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
42 |
struct |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
43 |
|
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
44 |
(** markup logical entities **) |
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
45 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
46 |
fun markup_class ctxt c = |
42379 | 47 |
[Name_Space.markup (Type.class_space (Proof_Context.tsig_of ctxt)) c]; |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
48 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
49 |
fun markup_type ctxt c = |
42379 | 50 |
[Name_Space.markup (Type.type_space (Proof_Context.tsig_of ctxt)) c]; |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
51 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
52 |
fun markup_const ctxt c = |
42379 | 53 |
[Name_Space.markup (Consts.space_of (Proof_Context.consts_of ctxt)) c]; |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
54 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
55 |
fun markup_free ctxt x = |
80746
fecfbcf41473
clarified markup: more uniform treatment of parse/print phase;
wenzelm
parents:
80745
diff
changeset
|
56 |
let |
fecfbcf41473
clarified markup: more uniform treatment of parse/print phase;
wenzelm
parents:
80745
diff
changeset
|
57 |
val m1 = |
fecfbcf41473
clarified markup: more uniform treatment of parse/print phase;
wenzelm
parents:
80745
diff
changeset
|
58 |
if Variable.is_fixed ctxt x then Variable.markup_fixed ctxt x |
fecfbcf41473
clarified markup: more uniform treatment of parse/print phase;
wenzelm
parents:
80745
diff
changeset
|
59 |
else if not (Variable.is_body ctxt) orelse Syntax.is_pretty_global ctxt then Markup.fixed x |
fecfbcf41473
clarified markup: more uniform treatment of parse/print phase;
wenzelm
parents:
80745
diff
changeset
|
60 |
else Markup.intensify; |
fecfbcf41473
clarified markup: more uniform treatment of parse/print phase;
wenzelm
parents:
80745
diff
changeset
|
61 |
val m2 = Variable.markup ctxt x; |
fecfbcf41473
clarified markup: more uniform treatment of parse/print phase;
wenzelm
parents:
80745
diff
changeset
|
62 |
in [m1, m2] end; |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
63 |
|
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
64 |
fun markup_var xi = [Markup.name (Term.string_of_vname xi) Markup.var]; |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
65 |
|
45412 | 66 |
fun markup_bound def ps (name, id) = |
74183 | 67 |
Markup.bound :: map (fn pos => Position.make_entity_markup def id Markup.boundN (name, pos)) ps; |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
68 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
69 |
fun markup_entity ctxt c = |
80748
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
70 |
Syntax.get_consts (Proof_Context.syntax_of ctxt) c |
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
71 |
|> maps (Lexicon.unmark |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
72 |
{case_class = markup_class ctxt, |
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
73 |
case_type = markup_type ctxt, |
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
74 |
case_const = markup_const ctxt, |
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
75 |
case_fixed = markup_free ctxt, |
80748
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
76 |
case_default = K []}); |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
77 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
78 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
79 |
|
63395 | 80 |
(** reports of implicit variable scope **) |
81 |
||
82 |
fun reports_of_scope [] = [] |
|
83 |
| reports_of_scope (def_pos :: ps) = |
|
84 |
let |
|
85 |
val id = serial (); |
|
74183 | 86 |
fun entity def = Position.make_entity_markup def id "" ("", def_pos); |
63395 | 87 |
in |
88 |
map (rpair Markup.bound) (def_pos :: ps) @ |
|
74262 | 89 |
((def_pos, entity {def = true}) :: map (rpair (entity {def = false})) ps) |
63395 | 90 |
end; |
91 |
||
92 |
||
93 |
||
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
94 |
(** decode parse trees **) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
95 |
|
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
96 |
(* decode_sort *) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
97 |
|
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
98 |
fun decode_sort tm = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
99 |
let |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
100 |
fun err () = raise TERM ("decode_sort: bad encoding of classes", [tm]); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
101 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
102 |
fun class s = Lexicon.unmark_class s handle Fail _ => err (); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
103 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
104 |
fun classes (Const (s, _)) = [class s] |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
105 |
| classes (Const ("_classes", _) $ Const (s, _) $ cs) = class s :: classes cs |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
106 |
| classes _ = err (); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
107 |
|
67718 | 108 |
fun sort (Const ("_dummy_sort", _)) = dummyS |
109 |
| sort (Const ("_topsort", _)) = [] |
|
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
110 |
| sort (Const ("_sort", _) $ cs) = classes cs |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
111 |
| sort (Const (s, _)) = [class s] |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
112 |
| sort _ = err (); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
113 |
in sort tm end; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
114 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
115 |
|
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
116 |
(* decode_typ *) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
117 |
|
49685
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
118 |
fun decode_pos (Free (s, _)) = |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
119 |
if is_some (Term_Position.decode s) then SOME s else NONE |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
120 |
| decode_pos _ = NONE; |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
121 |
|
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
122 |
fun decode_typ tm = |
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
123 |
let |
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
124 |
fun err () = raise TERM ("decode_typ: bad encoding of type", [tm]); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
125 |
|
49685
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
126 |
fun typ ps sort tm = |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
127 |
(case tm of |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
128 |
Const ("_tfree", _) $ t => typ ps sort t |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
129 |
| Const ("_tvar", _) $ t => typ ps sort t |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
130 |
| Const ("_ofsort", _) $ t $ s => |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
131 |
(case decode_pos s of |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
132 |
SOME p => typ (p :: ps) sort t |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
133 |
| NONE => |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
134 |
if is_none sort then typ ps (SOME (decode_sort s)) t |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
135 |
else err ()) |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
136 |
| Const ("_dummy_ofsort", _) $ s => TFree ("'_dummy_", decode_sort s) |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
137 |
| Free (x, _) => TFree (x, ps @ the_default dummyS sort) |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
138 |
| Var (xi, _) => TVar (xi, ps @ the_default dummyS sort) |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
139 |
| _ => |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
140 |
if null ps andalso is_none sort then |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
141 |
let |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
142 |
val (head, args) = Term.strip_comb tm; |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
143 |
val a = |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
144 |
(case head of |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
145 |
Const (c, _) => (Lexicon.unmark_type c handle Fail _ => err ()) |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
146 |
| _ => err ()); |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
147 |
in Type (a, map (typ [] NONE) args) end |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
148 |
else err ()); |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
149 |
in typ [] NONE tm end; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
150 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
151 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
152 |
(* parsetree_to_ast *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
153 |
|
52188 | 154 |
fun parsetree_to_ast ctxt trf parsetree = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
155 |
let |
55922
710bc66f432c
more markup for inner syntax class/type names (notably for completion);
wenzelm
parents:
55829
diff
changeset
|
156 |
val reports = Unsynchronized.ref ([]: Position.report_text list); |
44735 | 157 |
fun report pos = Position.store_reports reports [pos]; |
55959
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
158 |
val append_reports = Position.append_reports reports; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
159 |
|
73163
624c2b98860a
suppress markup for literal tokens with block control symbols, for better PIDE/HTML output (see also d15fe10593ff);
wenzelm
parents:
71675
diff
changeset
|
160 |
fun report_pos tok = |
624c2b98860a
suppress markup for literal tokens with block control symbols, for better PIDE/HTML output (see also d15fe10593ff);
wenzelm
parents:
71675
diff
changeset
|
161 |
if Lexicon.suppress_markup tok then Position.none |
624c2b98860a
suppress markup for literal tokens with block control symbols, for better PIDE/HTML output (see also d15fe10593ff);
wenzelm
parents:
71675
diff
changeset
|
162 |
else Lexicon.pos_of_token tok; |
624c2b98860a
suppress markup for literal tokens with block control symbols, for better PIDE/HTML output (see also d15fe10593ff);
wenzelm
parents:
71675
diff
changeset
|
163 |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
164 |
fun trans a args = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
165 |
(case trf a of |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
166 |
NONE => Ast.mk_appl (Ast.Constant a) args |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
167 |
| SOME f => f ctxt args); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
168 |
|
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
169 |
fun asts_of_token tok = |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
170 |
if Lexicon.valued_token tok |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
171 |
then [Ast.Variable (Lexicon.str_of_token tok)] |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
172 |
else []; |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
173 |
|
52162
896ebb4646d8
position constraint for dummy_pattern -- more PIDE markup;
wenzelm
parents:
52160
diff
changeset
|
174 |
fun ast_of_position tok = |
73163
624c2b98860a
suppress markup for literal tokens with block control symbols, for better PIDE/HTML output (see also d15fe10593ff);
wenzelm
parents:
71675
diff
changeset
|
175 |
Ast.Variable (Term_Position.encode (report_pos tok)); |
52162
896ebb4646d8
position constraint for dummy_pattern -- more PIDE markup;
wenzelm
parents:
52160
diff
changeset
|
176 |
|
52163
72e83c82c1d4
position constraint for bound dummy -- more PIDE markup;
wenzelm
parents:
52162
diff
changeset
|
177 |
fun ast_of_dummy a tok = |
52188 | 178 |
Ast.Appl [Ast.Constant "_constrain", Ast.Constant a, ast_of_position tok]; |
52163
72e83c82c1d4
position constraint for bound dummy -- more PIDE markup;
wenzelm
parents:
52162
diff
changeset
|
179 |
|
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
180 |
fun asts_of_position c tok = |
52188 | 181 |
[Ast.Appl [Ast.Constant c, ast_of (Parser.Tip tok), ast_of_position tok]] |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
182 |
|
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
183 |
and asts_of (Parser.Node ("_class_name", [Parser.Tip tok])) = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
184 |
let |
73163
624c2b98860a
suppress markup for literal tokens with block control symbols, for better PIDE/HTML output (see also d15fe10593ff);
wenzelm
parents:
71675
diff
changeset
|
185 |
val pos = report_pos tok; |
55922
710bc66f432c
more markup for inner syntax class/type names (notably for completion);
wenzelm
parents:
55829
diff
changeset
|
186 |
val (c, rs) = Proof_Context.check_class ctxt (Lexicon.str_of_token tok, pos); |
55959
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
187 |
val _ = append_reports rs; |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
188 |
in [Ast.Constant (Lexicon.mark_class c)] end |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
189 |
| asts_of (Parser.Node ("_type_name", [Parser.Tip tok])) = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
190 |
let |
73163
624c2b98860a
suppress markup for literal tokens with block control symbols, for better PIDE/HTML output (see also d15fe10593ff);
wenzelm
parents:
71675
diff
changeset
|
191 |
val pos = report_pos tok; |
55922
710bc66f432c
more markup for inner syntax class/type names (notably for completion);
wenzelm
parents:
55829
diff
changeset
|
192 |
val (Type (c, _), rs) = |
56002 | 193 |
Proof_Context.check_type_name {proper = true, strict = false} ctxt |
55951
c07d184aebe9
tuned signature -- more uniform check_type_name/read_type_name;
wenzelm
parents:
55950
diff
changeset
|
194 |
(Lexicon.str_of_token tok, pos); |
55959
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
195 |
val _ = append_reports rs; |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
196 |
in [Ast.Constant (Lexicon.mark_type c)] end |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
197 |
| asts_of (Parser.Node ("_position", [Parser.Tip tok])) = asts_of_position "_constrain" tok |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
198 |
| asts_of (Parser.Node ("_position_sort", [Parser.Tip tok])) = asts_of_position "_ofsort" tok |
62529
8b7bdfc09f3b
clarified treatment of fragments of Isabelle symbols during bootstrap;
wenzelm
parents:
62505
diff
changeset
|
199 |
| asts_of (Parser.Node (a as "\<^const>Pure.dummy_pattern", [Parser.Tip tok])) = |
52163
72e83c82c1d4
position constraint for bound dummy -- more PIDE markup;
wenzelm
parents:
52162
diff
changeset
|
200 |
[ast_of_dummy a tok] |
72e83c82c1d4
position constraint for bound dummy -- more PIDE markup;
wenzelm
parents:
52162
diff
changeset
|
201 |
| asts_of (Parser.Node (a as "_idtdummy", [Parser.Tip tok])) = |
72e83c82c1d4
position constraint for bound dummy -- more PIDE markup;
wenzelm
parents:
52162
diff
changeset
|
202 |
[ast_of_dummy a tok] |
72e83c82c1d4
position constraint for bound dummy -- more PIDE markup;
wenzelm
parents:
52162
diff
changeset
|
203 |
| asts_of (Parser.Node ("_idtypdummy", pts as [Parser.Tip tok, _, _])) = |
72e83c82c1d4
position constraint for bound dummy -- more PIDE markup;
wenzelm
parents:
52162
diff
changeset
|
204 |
[Ast.Appl (Ast.Constant "_constrain" :: ast_of_dummy "_idtdummy" tok :: maps asts_of pts)] |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
205 |
| asts_of (Parser.Node (a, pts)) = |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
206 |
let |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
207 |
val _ = pts |> List.app |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
208 |
(fn Parser.Node _ => () | Parser.Tip tok => |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
209 |
if Lexicon.valued_token tok then () |
73163
624c2b98860a
suppress markup for literal tokens with block control symbols, for better PIDE/HTML output (see also d15fe10593ff);
wenzelm
parents:
71675
diff
changeset
|
210 |
else report (report_pos tok) (markup_entity ctxt) a); |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
211 |
in [trans a (maps asts_of pts)] end |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
212 |
| asts_of (Parser.Tip tok) = asts_of_token tok |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
213 |
|
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
214 |
and ast_of pt = |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
215 |
(case asts_of pt of |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
216 |
[ast] => ast |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
217 |
| asts => raise Ast.AST ("parsetree_to_ast: malformed parsetree", asts)); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
218 |
|
78705
fde0b195cb7d
clarified signature: avoid association with potentially dangerous Exn.capture;
wenzelm
parents:
74571
diff
changeset
|
219 |
val ast = Exn.result ast_of parsetree; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
220 |
in (! reports, ast) end; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
221 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
222 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
223 |
(* ast_to_term *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
224 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
225 |
fun ast_to_term ctxt trf = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
226 |
let |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
227 |
fun trans a args = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
228 |
(case trf a of |
42476 | 229 |
NONE => Term.list_comb (Syntax.const a, args) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
230 |
| SOME f => f ctxt args); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
231 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
232 |
fun term_of (Ast.Constant a) = trans a [] |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
233 |
| term_of (Ast.Variable x) = Lexicon.read_var x |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
234 |
| term_of (Ast.Appl (Ast.Constant a :: (asts as _ :: _))) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
235 |
trans a (map term_of asts) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
236 |
| term_of (Ast.Appl (ast :: (asts as _ :: _))) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
237 |
Term.list_comb (term_of ast, map term_of asts) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
238 |
| term_of (ast as Ast.Appl _) = raise Ast.AST ("ast_to_term: malformed ast", [ast]); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
239 |
in term_of end; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
240 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
241 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
242 |
(* decode_term -- transform parse tree into raw term *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
243 |
|
55959
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
244 |
fun decode_const ctxt (c, ps) = |
55954 | 245 |
let |
55959
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
246 |
val (Const (c', _), reports) = |
56002 | 247 |
Proof_Context.check_const {proper = true, strict = false} ctxt (c, ps); |
55959
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
248 |
in (c', reports) end; |
55950
3bb5c7179234
clarified treatment of consts -- prefer value-oriented reports;
wenzelm
parents:
55949
diff
changeset
|
249 |
|
55976
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
250 |
local |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
251 |
|
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
252 |
fun get_free ctxt x = |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
253 |
let |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
254 |
val fixed = Variable.lookup_fixed ctxt x; |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
255 |
val is_const = can (decode_const ctxt) (x, []) orelse Long_Name.is_qualified x; |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
256 |
val is_declared = is_some (Variable.def_type ctxt false (x, ~1)); |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
257 |
in |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
258 |
if Variable.is_const ctxt x then NONE |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
259 |
else if is_some fixed then fixed |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
260 |
else if not is_const orelse is_declared then SOME x |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
261 |
else NONE |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
262 |
end; |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
263 |
|
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
264 |
in |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
265 |
|
55922
710bc66f432c
more markup for inner syntax class/type names (notably for completion);
wenzelm
parents:
55829
diff
changeset
|
266 |
fun decode_term _ (result as (_: Position.report_text list, Exn.Exn _)) = result |
43761
e72ba84ae58f
tuned signature -- corresponding to Scala version;
wenzelm
parents:
43731
diff
changeset
|
267 |
| decode_term ctxt (reports0, Exn.Res tm) = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
268 |
let |
55959
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
269 |
val reports = Unsynchronized.ref reports0; |
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
270 |
fun report ps = Position.store_reports reports ps; |
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
271 |
val append_reports = Position.append_reports reports; |
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
272 |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
273 |
fun decode ps qs bs (Const ("_constrain", _) $ t $ typ) = |
42264 | 274 |
(case Term_Position.decode_position typ of |
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
275 |
SOME (p, T) => Type.constraint T (decode (p :: ps) qs bs t) |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
276 |
| NONE => Type.constraint (decode_typ typ) (decode ps qs bs t)) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
277 |
| decode ps qs bs (Const ("_constrainAbs", _) $ t $ typ) = |
42264 | 278 |
(case Term_Position.decode_position typ of |
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
279 |
SOME (q, T) => Type.constraint (T --> dummyT) (decode ps (q :: qs) bs t) |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
280 |
| NONE => Type.constraint (decode_typ typ --> dummyT) (decode ps qs bs t)) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
281 |
| decode _ qs bs (Abs (x, T, t)) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
282 |
let |
45412 | 283 |
val id = serial (); |
74262 | 284 |
val _ = report qs (markup_bound {def = true} qs) (x, id); |
45412 | 285 |
in Abs (x, T, decode [] [] ((qs, (x, id)) :: bs) t) end |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
286 |
| decode _ _ bs (t $ u) = decode [] [] bs t $ decode [] [] bs u |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
287 |
| decode ps _ _ (Const (a, T)) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
288 |
(case try Lexicon.unmark_fixed a of |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
289 |
SOME x => (report ps (markup_free ctxt) x; Free (x, T)) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
290 |
| NONE => |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
291 |
let |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
292 |
val c = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
293 |
(case try Lexicon.unmark_const a of |
55976
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
294 |
SOME c => c |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
295 |
| NONE => #1 (decode_const ctxt (a, []))); |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
296 |
val _ = report ps (markup_const ctxt) c; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
297 |
in Const (c, T) end) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
298 |
| decode ps _ _ (Free (a, T)) = |
55956
94d384d621b0
reject internal term names outright, and complete consts instead;
wenzelm
parents:
55955
diff
changeset
|
299 |
((Name.reject_internal (a, ps) handle ERROR msg => |
94d384d621b0
reject internal term names outright, and complete consts instead;
wenzelm
parents:
55955
diff
changeset
|
300 |
error (msg ^ Proof_Context.consts_completion_message ctxt (a, ps))); |
55976
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
301 |
(case get_free ctxt a of |
55959
c3b458435f4f
more decisive commitment to get_free vs. the_const;
wenzelm
parents:
55957
diff
changeset
|
302 |
SOME x => (report ps (markup_free ctxt) x; Free (x, T)) |
55976
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
303 |
| NONE => |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
304 |
let |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
305 |
val (c, rs) = decode_const ctxt (a, ps); |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
306 |
val _ = append_reports rs; |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
307 |
in Const (c, T) end)) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
308 |
| decode ps _ _ (Var (xi, T)) = (report ps markup_var xi; Var (xi, T)) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
309 |
| decode ps _ bs (t as Bound i) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
310 |
(case try (nth bs) i of |
74262 | 311 |
SOME (qs, (x, id)) => (report ps (markup_bound {def = false} qs) (x, id); t) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
312 |
| NONE => t); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
313 |
|
78705
fde0b195cb7d
clarified signature: avoid association with potentially dangerous Exn.capture;
wenzelm
parents:
74571
diff
changeset
|
314 |
val tm' = Exn.result (fn () => decode [] [] [] tm) (); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
315 |
in (! reports, tm') end; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
316 |
|
55976
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
317 |
end; |
43815ee659bc
more basic const report (without completion) for known Const within syntax tree, which usually refers to special syntax (without proper @{const_syntax} markers);
wenzelm
parents:
55960
diff
changeset
|
318 |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
319 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
320 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
321 |
(** parse **) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
322 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
323 |
(* results *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
324 |
|
43761
e72ba84ae58f
tuned signature -- corresponding to Scala version;
wenzelm
parents:
43731
diff
changeset
|
325 |
fun proper_results results = map_filter (fn (y, Exn.Res x) => SOME (y, x) | _ => NONE) results; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
326 |
fun failed_results results = map_filter (fn (y, Exn.Exn e) => SOME (y, e) | _ => NONE) results; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
327 |
|
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
328 |
fun report_result ctxt pos ambig_msgs results = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
329 |
(case (proper_results results, failed_results results) of |
62505 | 330 |
([], (reports, exn) :: _) => (Context_Position.reports_text ctxt reports; Exn.reraise exn) |
55922
710bc66f432c
more markup for inner syntax class/type names (notably for completion);
wenzelm
parents:
55829
diff
changeset
|
331 |
| ([(reports, x)], _) => (Context_Position.reports_text ctxt reports; x) |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
332 |
| _ => |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
333 |
if null ambig_msgs then |
48992 | 334 |
error ("Parse error: ambiguous syntax" ^ Position.here pos) |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
335 |
else error (cat_lines ambig_msgs)); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
336 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
337 |
|
42249 | 338 |
(* parse raw asts *) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
339 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
340 |
fun parse_asts ctxt raw root (syms, pos) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
341 |
let |
80074
951c371c1cd9
clarified names: discontinue odd convention from 3 decades ago;
wenzelm
parents:
78705
diff
changeset
|
342 |
val syn = Proof_Context.syntax_of ctxt; |
42253 | 343 |
val ast_tr = Syntax.parse_ast_translation syn; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
344 |
|
42251 | 345 |
val toks = Syntax.tokenize syn raw syms; |
73163
624c2b98860a
suppress markup for literal tokens with block control symbols, for better PIDE/HTML output (see also d15fe10593ff);
wenzelm
parents:
71675
diff
changeset
|
346 |
val _ = Context_Position.reports ctxt (maps Lexicon.reports_of_token toks); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
347 |
|
45641 | 348 |
val pts = Syntax.parse syn root (filter Lexicon.is_proper toks) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
349 |
handle ERROR msg => |
55957
cffb46aea3d1
more compact Markup.markup_report: message body may consist of multiple elements;
wenzelm
parents:
55956
diff
changeset
|
350 |
error (msg ^ Markup.markup_report (implode (map (Lexicon.reported_token_range ctxt) toks))); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
351 |
val len = length pts; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
352 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
353 |
val limit = Config.get ctxt Syntax.ambiguity_limit; |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
354 |
val ambig_msgs = |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
355 |
if len <= 1 then [] |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
356 |
else |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
357 |
[cat_lines |
62800 | 358 |
(("Ambiguous input" ^ Position.here (Position.no_range_position pos) ^ |
55979
06cb126f30ba
tuned message: reveal ambiguity where Syntax_Phases.decode_term fails and thus reduces proper_results beforehand, e.g. term "f(x := y)" in ~~/src/HOL/Hoare/Hoare_Logic.thy;
wenzelm
parents:
55976
diff
changeset
|
359 |
" produces " ^ string_of_int len ^ " parse trees" ^ |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
360 |
(if len <= limit then "" else " (" ^ string_of_int limit ^ " displayed)") ^ ":") :: |
80950 | 361 |
map (Pretty.string_of o Pretty.item o Parser.pretty_parsetree) (take limit pts))]; |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
362 |
|
52188 | 363 |
in (ambig_msgs, map (parsetree_to_ast ctxt ast_tr) pts) end; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
364 |
|
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
365 |
fun parse_tree ctxt root input = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
366 |
let |
80074
951c371c1cd9
clarified names: discontinue odd convention from 3 decades ago;
wenzelm
parents:
78705
diff
changeset
|
367 |
val syn = Proof_Context.syntax_of ctxt; |
42253 | 368 |
val tr = Syntax.parse_translation syn; |
42255 | 369 |
val parse_rules = Syntax.parse_rules syn; |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
370 |
val (ambig_msgs, asts) = parse_asts ctxt false root input; |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
371 |
val results = |
61077
06cca32aa519
thread context for exceptions from forks, e.g. relevant when printing errors;
wenzelm
parents:
60490
diff
changeset
|
372 |
(map o apsnd o Exn.maps_res) |
78705
fde0b195cb7d
clarified signature: avoid association with potentially dangerous Exn.capture;
wenzelm
parents:
74571
diff
changeset
|
373 |
(Ast.normalize ctxt parse_rules #> Exn.result (ast_to_term ctxt tr)) asts; |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
374 |
in (ambig_msgs, results) end; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
375 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
376 |
|
42249 | 377 |
(* parse logical entities *) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
378 |
|
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
379 |
fun parse_failed ctxt pos msg kind = |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
380 |
cat_error msg ("Failed to parse " ^ kind ^ |
64677
8dc24130e8fe
more uniform treatment of "bad" like other messages (with serial number);
wenzelm
parents:
63395
diff
changeset
|
381 |
Markup.markup_report (Context_Position.reported_text ctxt pos (Markup.bad ()) "")); |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
382 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
383 |
fun parse_sort ctxt = |
59795 | 384 |
Syntax.parse_input ctxt Term_XML.Decode.sort Markup.language_sort |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
385 |
(fn (syms, pos) => |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
386 |
parse_tree ctxt "sort" (syms, pos) |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
387 |
|> uncurry (report_result ctxt pos) |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
388 |
|> decode_sort |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
389 |
|> Type.minimize_sort (Proof_Context.tsig_of ctxt) |
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
390 |
handle ERROR msg => parse_failed ctxt pos msg "sort"); |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
391 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
392 |
fun parse_typ ctxt = |
59795 | 393 |
Syntax.parse_input ctxt Term_XML.Decode.typ Markup.language_type |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
394 |
(fn (syms, pos) => |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
395 |
parse_tree ctxt "type" (syms, pos) |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
396 |
|> uncurry (report_result ctxt pos) |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
397 |
|> decode_typ |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
398 |
handle ERROR msg => parse_failed ctxt pos msg "type"); |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
399 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
400 |
fun parse_term is_prop ctxt = |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
401 |
let |
42281 | 402 |
val (markup, kind, root, constrain) = |
403 |
if is_prop |
|
55550 | 404 |
then (Markup.language_prop, "prop", "prop", Type.constraint propT) |
405 |
else (Markup.language_term, "term", Config.get ctxt Syntax.root, I); |
|
70784
799437173553
Term_XML.Encode/Decode.term uses Const "typargs";
wenzelm
parents:
69042
diff
changeset
|
406 |
val decode = constrain o Term_XML.Decode.term (Proof_Context.consts_of ctxt); |
42249 | 407 |
in |
59795 | 408 |
Syntax.parse_input ctxt decode markup |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
409 |
(fn (syms, pos) => |
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
410 |
let |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
411 |
val (ambig_msgs, results) = parse_tree ctxt root (syms, pos) ||> map (decode_term ctxt); |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
412 |
val parsed_len = length (proper_results results); |
42249 | 413 |
|
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
414 |
val ambiguity_warning = Config.get ctxt Syntax.ambiguity_warning; |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
415 |
val limit = Config.get ctxt Syntax.ambiguity_limit; |
42249 | 416 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
417 |
(*brute-force disambiguation via type-inference*) |
60490
9b28f446d9c5
more informative check: dummies are always allowed parse_term and should not lead to rejection here;
wenzelm
parents:
59795
diff
changeset
|
418 |
fun check t = |
9b28f446d9c5
more informative check: dummies are always allowed parse_term and should not lead to rejection here;
wenzelm
parents:
59795
diff
changeset
|
419 |
(Syntax.check_term (Proof_Context.allow_dummies ctxt) (constrain t); Exn.Res t) |
9b28f446d9c5
more informative check: dummies are always allowed parse_term and should not lead to rejection here;
wenzelm
parents:
59795
diff
changeset
|
420 |
handle exn as ERROR _ => Exn.Exn exn; |
42249 | 421 |
|
73686 | 422 |
fun par_map xs = Par_List.map' {name = "Syntax_Phases.parse_term", sequential = false} xs; |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
423 |
val results' = |
73686 | 424 |
if parsed_len > 1 then (grouped 10 par_map o apsnd o Exn.maps_res) check results |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
425 |
else results; |
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
426 |
val reports' = fst (hd results'); |
42249 | 427 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
428 |
val errs = map snd (failed_results results'); |
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
429 |
val checked = map snd (proper_results results'); |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
430 |
val checked_len = length checked; |
42249 | 431 |
|
52517 | 432 |
val pretty_term = Syntax.pretty_term (Config.put Printer.show_brackets true ctxt); |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
433 |
in |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
434 |
if checked_len = 0 then |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
435 |
report_result ctxt pos [] |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
436 |
[(reports', Exn.Exn (Exn.EXCEPTIONS (map ERROR ambig_msgs @ errs)))] |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
437 |
else if checked_len = 1 then |
56294
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
56243
diff
changeset
|
438 |
(if not (null ambig_msgs) andalso ambiguity_warning andalso |
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
56243
diff
changeset
|
439 |
Context_Position.is_visible ctxt then |
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
56243
diff
changeset
|
440 |
warning |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
441 |
(cat_lines (ambig_msgs @ |
55979
06cb126f30ba
tuned message: reveal ambiguity where Syntax_Phases.decode_term fails and thus reduces proper_results beforehand, e.g. term "f(x := y)" in ~~/src/HOL/Hoare/Hoare_Logic.thy;
wenzelm
parents:
55976
diff
changeset
|
442 |
["Fortunately, only one parse tree is well-formed and type-correct,\n\ |
06cb126f30ba
tuned message: reveal ambiguity where Syntax_Phases.decode_term fails and thus reduces proper_results beforehand, e.g. term "f(x := y)" in ~~/src/HOL/Hoare/Hoare_Logic.thy;
wenzelm
parents:
55976
diff
changeset
|
443 |
\but you may still want to disambiguate your grammar or your input."])) |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
444 |
else (); report_result ctxt pos [] results') |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
445 |
else |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
446 |
report_result ctxt pos [] |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
447 |
[(reports', Exn.Exn (ERROR (cat_lines (ambig_msgs @ |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
448 |
(("Ambiguous input\n" ^ string_of_int checked_len ^ " terms are type correct" ^ |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
449 |
(if checked_len <= limit then "" |
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
450 |
else " (" ^ string_of_int limit ^ " displayed)") ^ ":") :: |
52517 | 451 |
map (Pretty.string_of o Pretty.item o single o pretty_term) |
452 |
(take limit checked))))))] |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
453 |
end handle ERROR msg => parse_failed ctxt pos msg kind) |
42249 | 454 |
end; |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
455 |
|
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
456 |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
457 |
(* parse_ast_pattern *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
458 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
459 |
fun parse_ast_pattern ctxt (root, str) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
460 |
let |
80074
951c371c1cd9
clarified names: discontinue odd convention from 3 decades ago;
wenzelm
parents:
78705
diff
changeset
|
461 |
val syn = Proof_Context.syntax_of ctxt; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
462 |
|
55922
710bc66f432c
more markup for inner syntax class/type names (notably for completion);
wenzelm
parents:
55829
diff
changeset
|
463 |
val reports = Unsynchronized.ref ([]: Position.report_text list); |
52188 | 464 |
fun report ps = Position.store_reports reports ps; |
465 |
||
466 |
fun decode_const ps c = (report ps (markup_entity ctxt) c; Ast.Constant c); |
|
467 |
fun decode_var ps x = (report ps (fn () => [Markup.name x Markup.free]) (); Ast.Variable x); |
|
468 |
fun decode_appl ps asts = Ast.Appl (map (decode ps) asts) |
|
469 |
and decode ps (Ast.Constant c) = decode_const ps c |
|
470 |
| decode ps (Ast.Variable x) = |
|
80739 | 471 |
if Syntax.is_const syn x orelse Long_Name.is_qualified x |
52188 | 472 |
then decode_const ps x |
473 |
else decode_var ps x |
|
474 |
| decode ps (Ast.Appl (asts as (Ast.Constant c :: ast :: Ast.Variable x :: args))) = |
|
475 |
if member (op =) Term_Position.markers c then |
|
476 |
(case Term_Position.decode x of |
|
477 |
SOME p => Ast.mk_appl (decode (p :: ps) ast) (map (decode ps) args) |
|
478 |
| NONE => decode_appl ps asts) |
|
479 |
else decode_appl ps asts |
|
480 |
| decode ps (Ast.Appl asts) = decode_appl ps asts; |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
481 |
|
59795 | 482 |
val source = Syntax.read_input str; |
59064 | 483 |
val pos = Input.pos_of source; |
484 |
val syms = Input.source_explode source; |
|
52188 | 485 |
val ast = |
58978
e42da880c61e
more position information, e.g. relevant for errors in generated ML source;
wenzelm
parents:
58047
diff
changeset
|
486 |
parse_asts ctxt true root (syms, pos) |
e42da880c61e
more position information, e.g. relevant for errors in generated ML source;
wenzelm
parents:
58047
diff
changeset
|
487 |
|> uncurry (report_result ctxt pos) |
52188 | 488 |
|> decode []; |
55922
710bc66f432c
more markup for inner syntax class/type names (notably for completion);
wenzelm
parents:
55829
diff
changeset
|
489 |
val _ = Context_Position.reports_text ctxt (! reports); |
52188 | 490 |
in ast end; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
491 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
492 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
493 |
|
42245 | 494 |
(** encode parse trees **) |
495 |
||
496 |
(* term_of_sort *) |
|
497 |
||
498 |
fun term_of_sort S = |
|
499 |
let |
|
42476 | 500 |
val class = Syntax.const o Lexicon.mark_class; |
42245 | 501 |
|
502 |
fun classes [c] = class c |
|
42476 | 503 |
| classes (c :: cs) = Syntax.const "_classes" $ class c $ classes cs; |
42245 | 504 |
in |
67718 | 505 |
if S = dummyS then Syntax.const "_dummy_sort" |
506 |
else |
|
507 |
(case S of |
|
508 |
[] => Syntax.const "_topsort" |
|
509 |
| [c] => class c |
|
510 |
| cs => Syntax.const "_sort" $ classes cs) |
|
42245 | 511 |
end; |
512 |
||
513 |
||
514 |
(* term_of_typ *) |
|
515 |
||
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
516 |
fun term_of_typ ctxt ty = |
42245 | 517 |
let |
52210
0226035df99d
more explicit Printer.type_emphasis, depending on show_type_emphasis;
wenzelm
parents:
52188
diff
changeset
|
518 |
val show_sorts = Config.get ctxt show_sorts orelse Config.get ctxt show_markup; |
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
519 |
|
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
520 |
fun ofsort t raw_S = |
52210
0226035df99d
more explicit Printer.type_emphasis, depending on show_type_emphasis;
wenzelm
parents:
52188
diff
changeset
|
521 |
if show_sorts then |
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
522 |
let val S = #2 (Term_Position.decode_positionS raw_S) |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
523 |
in if S = dummyS then t else Syntax.const "_ofsort" $ t $ term_of_sort S end |
42245 | 524 |
else t; |
525 |
||
526 |
fun term_of (Type (a, Ts)) = |
|
42476 | 527 |
Term.list_comb (Syntax.const (Lexicon.mark_type a), map term_of Ts) |
42245 | 528 |
| term_of (TFree (x, S)) = |
42290
b1f544c84040
discontinued special treatment of structure Lexicon;
wenzelm
parents:
42289
diff
changeset
|
529 |
if is_some (Term_Position.decode x) then Syntax.free x |
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
530 |
else ofsort (Syntax.const "_tfree" $ Syntax.free x) S |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
531 |
| term_of (TVar (xi, S)) = ofsort (Syntax.const "_tvar" $ Syntax.var xi) S; |
42245 | 532 |
in term_of ty end; |
533 |
||
534 |
||
535 |
(* simple_ast_of *) |
|
536 |
||
537 |
fun simple_ast_of ctxt = |
|
538 |
let |
|
539 |
val tune_var = if Config.get ctxt show_question_marks then I else unprefix "?"; |
|
540 |
fun ast_of (Const (c, _)) = Ast.Constant c |
|
541 |
| ast_of (Free (x, _)) = Ast.Variable x |
|
542 |
| ast_of (Var (xi, _)) = Ast.Variable (tune_var (Term.string_of_vname xi)) |
|
543 |
| ast_of (t as _ $ _) = |
|
544 |
let val (f, args) = strip_comb t |
|
545 |
in Ast.mk_appl (ast_of f) (map ast_of args) end |
|
42408 | 546 |
| ast_of (Bound i) = Ast.Appl [Ast.Constant "_loose", Ast.Variable ("B." ^ string_of_int i)] |
42245 | 547 |
| ast_of (Abs _) = raise Fail "simple_ast_of: Abs"; |
548 |
in ast_of end; |
|
549 |
||
550 |
||
551 |
(* sort_to_ast and typ_to_ast *) |
|
552 |
||
553 |
fun ast_of_termT ctxt trf tm = |
|
554 |
let |
|
555 |
val ctxt' = Config.put show_sorts false ctxt; |
|
556 |
fun ast_of (t as Const ("_tfree", _) $ Free _) = simple_ast_of ctxt t |
|
557 |
| ast_of (t as Const ("_tvar", _) $ Var _) = simple_ast_of ctxt t |
|
558 |
| ast_of (Const (a, _)) = trans a [] |
|
559 |
| ast_of (t as _ $ _) = |
|
560 |
(case strip_comb t of |
|
561 |
(Const (a, _), args) => trans a args |
|
562 |
| (f, args) => Ast.Appl (map ast_of (f :: args))) |
|
563 |
| ast_of t = simple_ast_of ctxt t |
|
42254 | 564 |
and trans a args = ast_of (trf a ctxt' dummyT args) |
565 |
handle Match => Ast.mk_appl (Ast.Constant a) (map ast_of args); |
|
42245 | 566 |
in ast_of tm end; |
567 |
||
568 |
fun sort_to_ast ctxt trf S = ast_of_termT ctxt trf (term_of_sort S); |
|
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
569 |
fun typ_to_ast ctxt trf T = ast_of_termT ctxt trf (term_of_typ ctxt T); |
42245 | 570 |
|
571 |
||
572 |
(* term_to_ast *) |
|
573 |
||
52177 | 574 |
local |
575 |
||
576 |
fun mark_aprop tm = |
|
577 |
let |
|
578 |
fun aprop t = Syntax.const "_aprop" $ t; |
|
579 |
||
580 |
fun is_prop Ts t = |
|
52464
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
581 |
Type_Annotation.clean (Type_Annotation.fastype_of Ts t) = propT |
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
582 |
handle TERM _ => false; |
52177 | 583 |
|
584 |
fun is_term (Const ("Pure.term", _) $ _) = true |
|
585 |
| is_term _ = false; |
|
586 |
||
587 |
fun mark _ (t as Const _) = t |
|
588 |
| mark Ts (t as Const ("_bound", _) $ u) = if is_prop Ts u then aprop t else t |
|
52464
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
589 |
| mark Ts (t as Free _) = if is_prop Ts t then aprop t else t |
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
590 |
| mark Ts (t as Var _) = if is_prop Ts t then aprop t else t |
52177 | 591 |
| mark Ts (t as Bound _) = if is_prop Ts t then aprop t else t |
592 |
| mark Ts (Abs (x, T, t)) = Abs (x, T, mark (T :: Ts) t) |
|
56243 | 593 |
| mark Ts (t as t1 $ (t2 as Const ("Pure.type", Type ("itself", [T])))) = |
52177 | 594 |
if is_prop Ts t andalso not (is_term t) then Const ("_type_prop", T) $ mark Ts t1 |
595 |
else mark Ts t1 $ mark Ts t2 |
|
596 |
| mark Ts (t as t1 $ t2) = |
|
597 |
(if is_Const (Term.head_of t) orelse not (is_prop Ts t) then I else aprop) |
|
598 |
(mark Ts t1 $ mark Ts t2); |
|
599 |
in mark [] tm end; |
|
600 |
||
62239 | 601 |
fun prune_types tm = |
42245 | 602 |
let |
52211
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
603 |
fun regard t t' seen = |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
604 |
if Type_Annotation.is_omitted (Type_Annotation.fastype_of [] t) then (t, seen) |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
605 |
else if member (op aconv) seen t then (t', seen) |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
606 |
else (t, t :: seen); |
42245 | 607 |
|
52211
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
608 |
fun prune (t as Const _, seen) = (t, seen) |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
609 |
| prune (t as Free (x, T), seen) = regard t (Free (x, Type_Annotation.ignore_type T)) seen |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
610 |
| prune (t as Var (xi, T), seen) = regard t (Var (xi, Type_Annotation.ignore_type T)) seen |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
611 |
| prune (t as Bound _, seen) = (t, seen) |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
612 |
| prune (Abs (x, T, t), seen) = |
52186 | 613 |
let val (t', seen') = prune (t, seen); |
52211
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
614 |
in (Abs (x, T, t'), seen') end |
52186 | 615 |
| prune (t1 $ t2, seen) = |
52177 | 616 |
let |
52186 | 617 |
val (t1', seen') = prune (t1, seen); |
618 |
val (t2', seen'') = prune (t2, seen'); |
|
52177 | 619 |
in (t1' $ t2', seen'') end; |
52186 | 620 |
in #1 (prune (tm, [])) end; |
52177 | 621 |
|
80749 | 622 |
fun mark_atoms ctxt tm = |
52186 | 623 |
let |
59152
66e6c539a36d
more frugal Local_Syntax.init -- maintain idents within context;
wenzelm
parents:
59064
diff
changeset
|
624 |
val {structs, fixes} = Syntax_Trans.get_idents ctxt; |
52186 | 625 |
val show_structs = Config.get ctxt show_structs; |
626 |
||
627 |
fun mark ((t as Const (c, _)) $ u) = |
|
52160 | 628 |
if member (op =) Pure_Thy.token_markers c |
52186 | 629 |
then t $ u else mark t $ mark u |
630 |
| mark (t $ u) = mark t $ mark u |
|
631 |
| mark (Abs (x, T, t)) = Abs (x, T, mark t) |
|
632 |
| mark (t as Const (c, T)) = |
|
80749 | 633 |
if Proof_Context.is_syntax_const ctxt c then t |
42245 | 634 |
else Const (Lexicon.mark_const c, T) |
52186 | 635 |
| mark (t as Free (x, T)) = |
42245 | 636 |
let val i = find_index (fn s => s = x) structs + 1 in |
637 |
if i = 0 andalso member (op =) fixes x then |
|
638 |
Const (Lexicon.mark_fixed x, T) |
|
639 |
else if i = 1 andalso not show_structs then |
|
42476 | 640 |
Syntax.const "_struct" $ Syntax.const "_indexdefault" |
641 |
else Syntax.const "_free" $ t |
|
42245 | 642 |
end |
52186 | 643 |
| mark (t as Var (xi, T)) = |
62763 | 644 |
if xi = Auto_Bind.dddot then Const ("_DDDOT", T) |
42476 | 645 |
else Syntax.const "_var" $ t |
52186 | 646 |
| mark a = a; |
647 |
in mark tm end; |
|
648 |
||
649 |
in |
|
650 |
||
80740 | 651 |
fun term_to_ast ctxt trf tm = |
52186 | 652 |
let |
653 |
val show_types = Config.get ctxt show_types orelse Config.get ctxt show_sorts; |
|
654 |
val show_markup = Config.get ctxt show_markup; |
|
42245 | 655 |
|
656 |
fun ast_of tm = |
|
657 |
(case strip_comb tm of |
|
42284 | 658 |
(t as Abs _, ts) => Ast.mk_appl (ast_of (Syntax_Trans.abs_tr' ctxt t)) (map ast_of ts) |
42245 | 659 |
| ((c as Const ("_free", _)), Free (x, T) :: ts) => |
42290
b1f544c84040
discontinued special treatment of structure Lexicon;
wenzelm
parents:
42289
diff
changeset
|
660 |
Ast.mk_appl (constrain (c $ Syntax.free x) T) (map ast_of ts) |
42245 | 661 |
| ((c as Const ("_var", _)), Var (xi, T) :: ts) => |
42290
b1f544c84040
discontinued special treatment of structure Lexicon;
wenzelm
parents:
42289
diff
changeset
|
662 |
Ast.mk_appl (constrain (c $ Syntax.var xi) T) (map ast_of ts) |
49660
de49d9b4d7bc
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm
parents:
49659
diff
changeset
|
663 |
| ((c as Const ("_bound", B)), Free (x, T) :: ts) => |
de49d9b4d7bc
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm
parents:
49659
diff
changeset
|
664 |
let |
de49d9b4d7bc
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm
parents:
49659
diff
changeset
|
665 |
val X = |
de49d9b4d7bc
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm
parents:
49659
diff
changeset
|
666 |
if show_markup andalso not show_types orelse B <> dummyT then T |
de49d9b4d7bc
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm
parents:
49659
diff
changeset
|
667 |
else dummyT; |
de49d9b4d7bc
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm
parents:
49659
diff
changeset
|
668 |
in Ast.mk_appl (constrain (c $ Syntax.free x) X) (map ast_of ts) end |
42245 | 669 |
| (Const ("_idtdummy", T), ts) => |
42476 | 670 |
Ast.mk_appl (constrain (Syntax.const "_idtdummy") T) (map ast_of ts) |
62239 | 671 |
| (Const (c, T), ts) => trans c (Type_Annotation.smash T) ts |
42245 | 672 |
| (t, ts) => Ast.mk_appl (simple_ast_of ctxt t) (map ast_of ts)) |
673 |
||
42254 | 674 |
and trans a T args = ast_of (trf a ctxt T args) |
675 |
handle Match => Ast.mk_appl (Ast.Constant a) (map ast_of args) |
|
42245 | 676 |
|
52211
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
677 |
and constrain t T0 = |
52464
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
678 |
let |
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
679 |
val T = |
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
680 |
if show_markup andalso not show_types |
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
681 |
then Type_Annotation.clean T0 |
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
682 |
else Type_Annotation.smash T0; |
36497ee02ed8
clarified printing of type constraints vs. annotations, notably in goal display with its Type_Annotation.ignore_free_types;
wenzelm
parents:
52219
diff
changeset
|
683 |
in |
52211
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
684 |
if (show_types orelse show_markup) andalso T <> dummyT then |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
685 |
Ast.Appl [Ast.Constant "_constrain", simple_ast_of ctxt t, |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
686 |
ast_of_termT ctxt trf (term_of_typ ctxt T)] |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
687 |
else simple_ast_of ctxt t |
66bc827e37f8
explicit support for type annotations within printed syntax trees;
wenzelm
parents:
52210
diff
changeset
|
688 |
end; |
42245 | 689 |
in |
690 |
tm |
|
52177 | 691 |
|> mark_aprop |
62239 | 692 |
|> show_types ? prune_types |
55014
a93f496f6c30
general notion of auxiliary bounds within context;
wenzelm
parents:
53171
diff
changeset
|
693 |
|> Variable.revert_bounds ctxt |
80749 | 694 |
|> mark_atoms ctxt |
42245 | 695 |
|> ast_of |
696 |
end; |
|
697 |
||
52177 | 698 |
end; |
699 |
||
42245 | 700 |
|
701 |
||
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
702 |
(** unparse **) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
703 |
|
42245 | 704 |
local |
705 |
||
80743 | 706 |
fun extern_fixed ctxt x = |
707 |
if Name.is_skolem x then Variable.revert_fixed ctxt x else x; |
|
708 |
||
709 |
fun extern ctxt c = |
|
80748
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
710 |
(case Syntax.get_consts (Proof_Context.syntax_of ctxt) c of |
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
711 |
[b] => b |
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
712 |
| bs => |
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
713 |
(case filter Lexicon.is_marked bs of |
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
714 |
[] => c |
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
715 |
| [b] => b |
43c4817375bf
support for syntax const dependencies, with minimal integrity checks;
wenzelm
parents:
80747
diff
changeset
|
716 |
| _ => error ("Multiple logical entities for " ^ quote c ^ ": " ^ commas_quote bs))) |
80743 | 717 |
|> Lexicon.unmark |
718 |
{case_class = Proof_Context.extern_class ctxt, |
|
719 |
case_type = Proof_Context.extern_type ctxt, |
|
720 |
case_const = Proof_Context.extern_const ctxt, |
|
721 |
case_fixed = extern_fixed ctxt, |
|
722 |
case_default = I}; |
|
723 |
||
80746
fecfbcf41473
clarified markup: more uniform treatment of parse/print phase;
wenzelm
parents:
80745
diff
changeset
|
724 |
fun free_or_skolem ctxt x = (markup_free ctxt x, extern_fixed ctxt x); |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
725 |
|
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
726 |
fun var_or_skolem s = |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
727 |
(case Lexicon.read_variable s of |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
728 |
SOME (x, i) => |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
729 |
(case try Name.dest_skolem x of |
80745 | 730 |
SOME x' => (Markup.skolem, Term.string_of_vname (x', i)) |
731 |
| NONE => (Markup.var, s)) |
|
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
732 |
| NONE => (Markup.var, s)); |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
733 |
|
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
734 |
val typing_elem = YXML.output_markup_elem Markup.typing; |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
735 |
val sorting_elem = YXML.output_markup_elem Markup.sorting; |
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
736 |
|
80747 | 737 |
fun unparse_t t_to_ast prt_t markup ctxt t = |
42245 | 738 |
let |
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
739 |
val show_markup = Config.get ctxt show_markup; |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
740 |
val show_sorts = Config.get ctxt show_sorts; |
52185 | 741 |
val show_types = Config.get ctxt show_types orelse show_sorts; |
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
742 |
|
80074
951c371c1cd9
clarified names: discontinue odd convention from 3 decades ago;
wenzelm
parents:
78705
diff
changeset
|
743 |
val syn = Proof_Context.syntax_of ctxt; |
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
744 |
val prtabs = Syntax.prtabs syn; |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
745 |
val trf = Syntax.print_ast_translation syn; |
80747 | 746 |
val markup_extern = (markup_entity ctxt, extern ctxt); |
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
747 |
|
80882
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
748 |
val cache1 = Unsynchronized.ref (Ast.Table.empty: Markup.output Pretty.block Ast.Table.table); |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
749 |
val cache2 = Unsynchronized.ref (Ast.Table.empty: Markup.output Pretty.block Ast.Table.table); |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
750 |
|
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
751 |
fun token_trans "_tfree" x = SOME (Pretty.mark_str (Markup.tfree, x)) |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
752 |
| token_trans "_tvar" x = SOME (Pretty.mark_str (Markup.tvar, x)) |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
753 |
| token_trans "_free" x = SOME (Pretty.marks_str (free_or_skolem ctxt x)) |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
754 |
| token_trans "_bound" x = SOME (Pretty.mark_str (Markup.bound, x)) |
64677
8dc24130e8fe
more uniform treatment of "bad" like other messages (with serial number);
wenzelm
parents:
63395
diff
changeset
|
755 |
| token_trans "_loose" x = SOME (Pretty.mark_str (Markup.bad (), x)) |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
756 |
| token_trans "_var" x = SOME (Pretty.mark_str (var_or_skolem x)) |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
757 |
| token_trans "_numeral" x = SOME (Pretty.mark_str (Markup.numeral, x)) |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
758 |
| token_trans "_inner_string" x = SOME (Pretty.mark_str (Markup.inner_string, x)) |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
759 |
| token_trans _ _ = NONE; |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
760 |
|
49655 | 761 |
fun markup_trans a [Ast.Variable x] = token_trans a x |
49662
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
762 |
| markup_trans "_constrain" [t, ty] = constrain_trans t ty |
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
763 |
| markup_trans "_idtyp" [t, ty] = constrain_trans t ty |
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
764 |
| markup_trans "_ofsort" [ty, s] = ofsort_trans ty s |
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
765 |
| markup_trans _ _ = NONE |
49655 | 766 |
|
49662
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
767 |
and constrain_trans t ty = |
80879 | 768 |
if show_markup andalso not show_types |
80880 | 769 |
then SOME (markup_ast true t ty) else NONE |
49662
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
770 |
|
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
771 |
and ofsort_trans ty s = |
80879 | 772 |
if show_markup andalso not show_sorts |
80880 | 773 |
then SOME (markup_ast false ty s) else NONE |
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
774 |
|
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
775 |
and pretty_typ_ast m ast = ast |
80747 | 776 |
|> Printer.pretty_typ_ast ctxt prtabs trf markup_trans markup_extern |
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
777 |
|> Pretty.markup m |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
778 |
|
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
779 |
and pretty_ast m ast = ast |
80747 | 780 |
|> prt_t ctxt prtabs trf markup_trans markup_extern |
80848
df85df6315af
clarified signature: prefer explicit type Bytes.T;
wenzelm
parents:
80789
diff
changeset
|
781 |
|> Pretty.markup m |
df85df6315af
clarified signature: prefer explicit type Bytes.T;
wenzelm
parents:
80789
diff
changeset
|
782 |
|
80880 | 783 |
and markup_ast is_typing a A = |
80882
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
784 |
Pretty.make_block (markup_block is_typing A) |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
785 |
[(if is_typing then pretty_ast else pretty_typ_ast) Markup.empty a] |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
786 |
|
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
787 |
and markup_block is_typing A = |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
788 |
let val cache = if is_typing then cache1 else cache2 in |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
789 |
(case Ast.Table.lookup (! cache) A of |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
790 |
SOME block => block |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
791 |
| NONE => |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
792 |
let |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
793 |
val ((bg1, bg2), en) = if is_typing then typing_elem else sorting_elem; |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
794 |
val B = Pretty.symbolic_output (pretty_typ_ast Markup.empty A); |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
795 |
val bg = implode (bg1 :: Bytes.contents B @ [bg2]); |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
796 |
val block = {markup = (bg, en), consistent = false, indent = 0}; |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
797 |
in Unsynchronized.change cache (Ast.Table.update (A, block)); block end) |
2cdb00f797b1
performance tuning: cache for highly redundant markup (types and sorts);
wenzelm
parents:
80880
diff
changeset
|
798 |
end; |
42245 | 799 |
in |
42255 | 800 |
t_to_ast ctxt (Syntax.print_translation syn) t |
801 |
|> Ast.normalize ctxt (Syntax.print_rules syn) |
|
80747 | 802 |
|> pretty_ast markup |
42245 | 803 |
end; |
804 |
||
805 |
in |
|
806 |
||
55828
42ac3cfb89f6
clarified language markup: added "delimited" property;
wenzelm
parents:
55550
diff
changeset
|
807 |
val unparse_sort = unparse_t sort_to_ast Printer.pretty_typ_ast (Markup.language_sort false); |
42ac3cfb89f6
clarified language markup: added "delimited" property;
wenzelm
parents:
55550
diff
changeset
|
808 |
val unparse_typ = unparse_t typ_to_ast Printer.pretty_typ_ast (Markup.language_type false); |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
809 |
|
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
810 |
fun unparse_term ctxt = |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
811 |
let |
42360 | 812 |
val thy = Proof_Context.theory_of ctxt; |
80740 | 813 |
val curried = not (Pure_Thy.old_appl_syntax thy); |
814 |
in unparse_t term_to_ast (Printer.pretty_term_ast curried) (Markup.language_term false) ctxt end; |
|
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
815 |
|
42249 | 816 |
end; |
817 |
||
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
818 |
|
42245 | 819 |
|
820 |
(** translations **) |
|
821 |
||
822 |
(* type propositions *) |
|
823 |
||
62529
8b7bdfc09f3b
clarified treatment of fragments of Isabelle symbols during bootstrap;
wenzelm
parents:
62505
diff
changeset
|
824 |
fun type_prop_tr' ctxt T [Const ("\<^const>Pure.sort_constraint", _)] = |
42476 | 825 |
Syntax.const "_sort_constraint" $ term_of_typ (Config.put show_sorts true ctxt) T |
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
826 |
| type_prop_tr' ctxt T [t] = |
42476 | 827 |
Syntax.const "_ofclass" $ term_of_typ ctxt T $ t |
42245 | 828 |
| type_prop_tr' _ T ts = raise TYPE ("type_prop_tr'", [T], ts); |
829 |
||
830 |
||
831 |
(* type reflection *) |
|
832 |
||
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
833 |
fun type_tr' ctxt (Type ("itself", [T])) ts = |
42476 | 834 |
Term.list_comb (Syntax.const "_TYPE" $ term_of_typ ctxt T, ts) |
42245 | 835 |
| type_tr' _ _ _ = raise Match; |
836 |
||
837 |
||
838 |
(* type constraints *) |
|
839 |
||
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
840 |
fun type_constraint_tr' ctxt (Type ("fun", [T, _])) (t :: ts) = |
42476 | 841 |
Term.list_comb (Syntax.const "_constrain" $ t $ term_of_typ ctxt T, ts) |
42245 | 842 |
| type_constraint_tr' _ _ _ = raise Match; |
843 |
||
844 |
||
42295
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
845 |
(* authentic syntax *) |
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
846 |
|
55960
beef468837b1
proper position for decode_pos, which is relevant for completion;
wenzelm
parents:
55959
diff
changeset
|
847 |
fun const_ast_tr intern ctxt asts = |
beef468837b1
proper position for decode_pos, which is relevant for completion;
wenzelm
parents:
55959
diff
changeset
|
848 |
(case asts of |
beef468837b1
proper position for decode_pos, which is relevant for completion;
wenzelm
parents:
55959
diff
changeset
|
849 |
[Ast.Appl [Ast.Constant "_constrain", Ast.Variable c, T as Ast.Variable p]] => |
42295
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
850 |
let |
55960
beef468837b1
proper position for decode_pos, which is relevant for completion;
wenzelm
parents:
55959
diff
changeset
|
851 |
val pos = the_default Position.none (Term_Position.decode p); |
beef468837b1
proper position for decode_pos, which is relevant for completion;
wenzelm
parents:
55959
diff
changeset
|
852 |
val (c', _) = decode_const ctxt (c, [pos]); |
42295
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
853 |
val d = if intern then Lexicon.mark_const c' else c; |
55960
beef468837b1
proper position for decode_pos, which is relevant for completion;
wenzelm
parents:
55959
diff
changeset
|
854 |
in Ast.Appl [Ast.Constant "_constrain", Ast.Constant d, T] end |
beef468837b1
proper position for decode_pos, which is relevant for completion;
wenzelm
parents:
55959
diff
changeset
|
855 |
| _ => raise Ast.AST ("const_ast_tr", asts)); |
42295
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
856 |
|
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
857 |
|
42245 | 858 |
(* setup translations *) |
859 |
||
53171 | 860 |
val _ = Theory.setup |
52143 | 861 |
(Sign.parse_ast_translation |
862 |
[("_context_const", const_ast_tr true), |
|
863 |
("_context_xconst", const_ast_tr false)] #> |
|
864 |
Sign.typed_print_translation |
|
42245 | 865 |
[("_type_prop", type_prop_tr'), |
62529
8b7bdfc09f3b
clarified treatment of fragments of Isabelle symbols during bootstrap;
wenzelm
parents:
62505
diff
changeset
|
866 |
("\<^const>Pure.type", type_tr'), |
53171 | 867 |
("_type_constraint_", type_constraint_tr')]); |
42245 | 868 |
|
869 |
||
870 |
||
42382
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
871 |
(** check/uncheck **) |
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
872 |
|
45429 | 873 |
(* context-sensitive (un)checking *) |
874 |
||
875 |
type key = int * bool; |
|
876 |
||
877 |
structure Checks = Generic_Data |
|
878 |
( |
|
879 |
type 'a check = 'a list -> Proof.context -> ('a list * Proof.context) option; |
|
880 |
type T = |
|
881 |
((key * ((string * typ check) * stamp) list) list * |
|
882 |
(key * ((string * term check) * stamp) list) list); |
|
883 |
val empty = ([], []); |
|
884 |
fun merge ((typ_checks1, term_checks1), (typ_checks2, term_checks2)) : T = |
|
885 |
(AList.join (op =) (K (Library.merge (eq_snd (op =)))) (typ_checks1, typ_checks2), |
|
886 |
AList.join (op =) (K (Library.merge (eq_snd (op =)))) (term_checks1, term_checks2)); |
|
887 |
); |
|
888 |
||
889 |
fun print_checks ctxt = |
|
890 |
let |
|
891 |
fun split_checks checks = |
|
892 |
List.partition (fn ((_, un), _) => not un) checks |
|
59058
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58978
diff
changeset
|
893 |
|> apply2 (map (fn ((i, _), fs) => (i, map (fst o fst) fs)) |
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58978
diff
changeset
|
894 |
#> sort (int_ord o apply2 fst)); |
45429 | 895 |
fun pretty_checks kind checks = |
896 |
checks |> map (fn (i, names) => Pretty.block |
|
897 |
[Pretty.str (kind ^ " (stage " ^ signed_string_of_int i ^ "):"), |
|
898 |
Pretty.brk 1, Pretty.strs names]); |
|
899 |
||
900 |
val (typs, terms) = Checks.get (Context.Proof ctxt); |
|
901 |
val (typ_checks, typ_unchecks) = split_checks typs; |
|
902 |
val (term_checks, term_unchecks) = split_checks terms; |
|
903 |
in |
|
904 |
pretty_checks "typ_checks" typ_checks @ |
|
905 |
pretty_checks "term_checks" term_checks @ |
|
906 |
pretty_checks "typ_unchecks" typ_unchecks @ |
|
907 |
pretty_checks "term_unchecks" term_unchecks |
|
56334
6b3739fee456
some shortcuts for chunks, which sometimes avoid bulky string output;
wenzelm
parents:
56333
diff
changeset
|
908 |
end |> Pretty.writeln_chunks; |
45429 | 909 |
|
910 |
||
911 |
local |
|
912 |
||
913 |
fun context_check which (key: key) name f = |
|
914 |
Checks.map (which (AList.map_default op = (key, []) (cons ((name, f), stamp ())))); |
|
915 |
||
916 |
fun simple_check eq f xs ctxt = |
|
917 |
let val xs' = f ctxt xs |
|
918 |
in if eq_list eq (xs, xs') then NONE else SOME (xs', ctxt) end; |
|
919 |
||
920 |
in |
|
921 |
||
45444 | 922 |
fun typ_check' stage = context_check apfst (stage, false); |
923 |
fun term_check' stage = context_check apsnd (stage, false); |
|
924 |
fun typ_uncheck' stage = context_check apfst (stage, true); |
|
925 |
fun term_uncheck' stage = context_check apsnd (stage, true); |
|
45429 | 926 |
|
45444 | 927 |
fun typ_check key name f = typ_check' key name (simple_check (op =) f); |
928 |
fun term_check key name f = term_check' key name (simple_check (op aconv) f); |
|
929 |
fun typ_uncheck key name f = typ_uncheck' key name (simple_check (op =) f); |
|
930 |
fun term_uncheck key name f = term_uncheck' key name (simple_check (op aconv) f); |
|
45429 | 931 |
|
932 |
end; |
|
933 |
||
934 |
||
935 |
local |
|
936 |
||
937 |
fun check_stage fs = perhaps_loop (perhaps_apply (map uncurry fs)); |
|
938 |
fun check_all fs = perhaps_apply (map check_stage fs); |
|
939 |
||
940 |
fun check which uncheck ctxt0 xs0 = |
|
941 |
let |
|
942 |
val funs = which (Checks.get (Context.Proof ctxt0)) |
|
943 |
|> map_filter (fn ((i, u), fs) => if uncheck = u then SOME (i, map (snd o fst) fs) else NONE) |
|
59058
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58978
diff
changeset
|
944 |
|> Library.sort (int_ord o apply2 fst) |> map snd |
45429 | 945 |
|> not uncheck ? map rev; |
946 |
in #1 (perhaps (check_all funs) (xs0, ctxt0)) end; |
|
947 |
||
948 |
val apply_typ_check = check fst false; |
|
949 |
val apply_term_check = check snd false; |
|
950 |
val apply_typ_uncheck = check fst true; |
|
951 |
val apply_term_uncheck = check snd true; |
|
952 |
||
953 |
in |
|
954 |
||
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
955 |
fun check_typs ctxt raw_tys = |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
956 |
let |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
957 |
val (sorting_report, tys) = Proof_Context.prepare_sortsT ctxt raw_tys; |
71675 | 958 |
val _ = if Context_Position.reports_enabled ctxt then Output.report sorting_report else (); |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
959 |
in |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
960 |
tys |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
961 |
|> apply_typ_check ctxt |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
962 |
|> Term_Sharing.typs (Proof_Context.theory_of ctxt) |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
963 |
end; |
45423
92f91f990165
tuned signature -- emphasize internal role of these operations;
wenzelm
parents:
45412
diff
changeset
|
964 |
|
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
965 |
fun check_terms ctxt raw_ts = |
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
966 |
let |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
967 |
val (sorting_report, raw_ts') = Proof_Context.prepare_sorts ctxt raw_ts; |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
968 |
val (ts, ps) = Type_Infer_Context.prepare_positions ctxt raw_ts'; |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
969 |
|
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
970 |
val tys = map (Logic.mk_type o snd) ps; |
45448
018f8959c7a6
more efficient prepare_sorts -- bypass encoded positions;
wenzelm
parents:
45447
diff
changeset
|
971 |
val (ts', tys') = ts @ tys |
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
972 |
|> apply_term_check ctxt |
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
973 |
|> chop (length ts); |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
974 |
val typing_report = |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
975 |
fold2 (fn (pos, _) => fn ty => |
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
976 |
if Position.is_reported pos then |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
977 |
cons (Position.reported_text pos Markup.typing |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
978 |
(Syntax.string_of_typ ctxt (Logic.dest_type ty))) |
56333
38f1422ef473
support bulk messages consisting of small string segments, which are more healthy to the Poly/ML RTS and might prevent spurious GC crashes such as MTGCProcessMarkPointers::ScanAddressesInObject;
wenzelm
parents:
56294
diff
changeset
|
979 |
else I) ps tys' []; |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
980 |
|
56294
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
56243
diff
changeset
|
981 |
val _ = |
71675 | 982 |
if Context_Position.reports_enabled ctxt |
983 |
then Output.report (sorting_report @ typing_report) else (); |
|
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
984 |
in Term_Sharing.terms (Proof_Context.theory_of ctxt) ts' end; |
45423
92f91f990165
tuned signature -- emphasize internal role of these operations;
wenzelm
parents:
45412
diff
changeset
|
985 |
|
42382
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
986 |
fun check_props ctxt = map (Type.constraint propT) #> check_terms ctxt; |
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
987 |
|
45429 | 988 |
val uncheck_typs = apply_typ_uncheck; |
989 |
val uncheck_terms = apply_term_uncheck; |
|
990 |
||
991 |
end; |
|
992 |
||
993 |
||
62952 | 994 |
(* install operations *) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
995 |
|
62897
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
996 |
val _ = |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
997 |
Theory.setup |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
998 |
(Syntax.install_operations |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
999 |
{parse_sort = parse_sort, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1000 |
parse_typ = parse_typ, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1001 |
parse_term = parse_term false, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1002 |
parse_prop = parse_term true, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1003 |
unparse_sort = unparse_sort, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1004 |
unparse_typ = unparse_typ, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1005 |
unparse_term = unparse_term, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1006 |
check_typs = check_typs, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1007 |
check_terms = check_terms, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1008 |
check_props = check_props, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1009 |
uncheck_typs = uncheck_typs, |
8093203f0b89
prefer regular context update, to allow continuous editing of Pure;
wenzelm
parents:
62800
diff
changeset
|
1010 |
uncheck_terms = uncheck_terms}); |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
1011 |
|
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
1012 |
end; |
62952 | 1013 |
|
1014 |
||
1015 |
(* standard phases *) |
|
1016 |
||
1017 |
val _ = Context.>> |
|
1018 |
(Syntax_Phases.typ_check 0 "standard" Proof_Context.standard_typ_check #> |
|
1019 |
Syntax_Phases.term_check 0 "standard" |
|
1020 |
(fn ctxt => Type_Infer_Context.infer_types ctxt #> map (Proof_Context.expand_abbrevs ctxt)) #> |
|
1021 |
Syntax_Phases.term_check 100 "standard_finish" Proof_Context.standard_term_check_finish #> |
|
1022 |
Syntax_Phases.term_uncheck 0 "standard" Proof_Context.standard_term_uncheck); |