author | wenzelm |
Thu, 03 Jan 2013 14:12:12 +0100 | |
changeset 50700 | e1df173b12a1 |
parent 50201 | c26369c9eda6 |
child 52143 | 36ffe23b25f8 |
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 |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
10 |
val decode_sort: term -> sort |
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
11 |
val decode_typ: term -> typ |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
12 |
val decode_term: Proof.context -> |
44736 | 13 |
Position.report list * term Exn.result -> Position.report list * term Exn.result |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
14 |
val parse_ast_pattern: Proof.context -> string * string -> Ast.ast |
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
15 |
val term_of_typ: Proof.context -> typ -> term |
45429 | 16 |
val print_checks: Proof.context -> unit |
17 |
val typ_check: int -> string -> (Proof.context -> typ list -> typ list) -> |
|
18 |
Context.generic -> Context.generic |
|
19 |
val term_check: int -> string -> (Proof.context -> term list -> term list) -> |
|
20 |
Context.generic -> Context.generic |
|
21 |
val typ_uncheck: int -> string -> (Proof.context -> typ list -> typ list) -> |
|
22 |
Context.generic -> Context.generic |
|
23 |
val term_uncheck: int -> string -> (Proof.context -> term list -> term list) -> |
|
24 |
Context.generic -> Context.generic |
|
45444 | 25 |
val typ_check': int -> string -> |
26 |
(typ list -> Proof.context -> (typ list * Proof.context) option) -> |
|
27 |
Context.generic -> Context.generic |
|
28 |
val term_check': int -> string -> |
|
29 |
(term list -> Proof.context -> (term list * Proof.context) option) -> |
|
30 |
Context.generic -> Context.generic |
|
31 |
val typ_uncheck': int -> string -> |
|
32 |
(typ list -> Proof.context -> (typ list * Proof.context) option) -> |
|
33 |
Context.generic -> Context.generic |
|
34 |
val term_uncheck': int -> string -> |
|
35 |
(term list -> Proof.context -> (term list * Proof.context) option) -> |
|
36 |
Context.generic -> Context.generic |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
37 |
end |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
38 |
|
42243 | 39 |
structure Syntax_Phases: SYNTAX_PHASES = |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
40 |
struct |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
41 |
|
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
42 |
(** 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
|
43 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
44 |
fun markup_class ctxt c = |
42379 | 45 |
[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
|
46 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
47 |
fun markup_type ctxt c = |
42379 | 48 |
[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
|
49 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
50 |
fun markup_const ctxt c = |
42379 | 51 |
[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
|
52 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
53 |
fun markup_free ctxt x = |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
54 |
[if can Name.dest_skolem x then Markup.skolem else Markup.free] @ |
42493
01430341fc79
more informative markup for fixed variables (via name space entry);
wenzelm
parents:
42488
diff
changeset
|
55 |
(if Variable.is_body ctxt orelse Variable.is_fixed ctxt x |
01430341fc79
more informative markup for fixed variables (via name space entry);
wenzelm
parents:
42488
diff
changeset
|
56 |
then [Variable.markup_fixed ctxt x] |
01430341fc79
more informative markup for fixed variables (via name space entry);
wenzelm
parents:
42488
diff
changeset
|
57 |
else []); |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
58 |
|
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
59 |
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
|
60 |
|
45412 | 61 |
fun markup_bound def ps (name, id) = |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
62 |
let val entity = Markup.entity Markup.boundN name in |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
63 |
Markup.bound :: |
45412 | 64 |
map (fn pos => Markup.properties (Position.entity_properties_of def id pos) entity) ps |
65 |
end; |
|
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
66 |
|
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
67 |
fun markup_entity ctxt c = |
42360 | 68 |
(case Syntax.lookup_const (Proof_Context.syn_of ctxt) c of |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
69 |
SOME "" => [] |
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
70 |
| SOME b => markup_entity ctxt b |
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
71 |
| NONE => c |> Lexicon.unmark |
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, |
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
76 |
case_default = K []}); |
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 |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
80 |
(** decode parse trees **) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
81 |
|
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
82 |
(* decode_sort *) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
83 |
|
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
84 |
fun decode_sort tm = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
85 |
let |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
86 |
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
|
87 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
88 |
fun class s = Lexicon.unmark_class s handle Fail _ => err (); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
89 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
90 |
fun classes (Const (s, _)) = [class s] |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
91 |
| classes (Const ("_classes", _) $ Const (s, _) $ cs) = class s :: classes cs |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
92 |
| classes _ = err (); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
93 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
94 |
fun sort (Const ("_topsort", _)) = [] |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
95 |
| sort (Const ("_sort", _) $ cs) = classes cs |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
96 |
| sort (Const (s, _)) = [class s] |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
97 |
| sort _ = err (); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
98 |
in sort tm end; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
99 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
100 |
|
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
101 |
(* decode_typ *) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
102 |
|
49685
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
103 |
fun decode_pos (Free (s, _)) = |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
104 |
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
|
105 |
| decode_pos _ = NONE; |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
106 |
|
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
107 |
fun decode_typ tm = |
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
108 |
let |
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
109 |
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
|
110 |
|
49685
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
111 |
fun typ ps sort tm = |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
112 |
(case tm of |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
113 |
Const ("_tfree", _) $ t => typ ps sort t |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
114 |
| Const ("_tvar", _) $ t => typ ps sort t |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
115 |
| Const ("_ofsort", _) $ t $ s => |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
116 |
(case decode_pos s of |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
117 |
SOME p => typ (p :: ps) sort t |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
118 |
| NONE => |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
119 |
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
|
120 |
else err ()) |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
121 |
| 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
|
122 |
| 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
|
123 |
| 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
|
124 |
| _ => |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
125 |
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
|
126 |
let |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
127 |
val (head, args) = Term.strip_comb tm; |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
128 |
val a = |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
129 |
(case head of |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
130 |
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
|
131 |
| _ => err ()); |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
132 |
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
|
133 |
else err ()); |
4341e4d86872
allow position constraints to coexist with 0 or 1 sort constraints;
wenzelm
parents:
49674
diff
changeset
|
134 |
in typ [] NONE tm end; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
135 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
136 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
137 |
(* parsetree_to_ast *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
138 |
|
46126
bab00660539d
discontinued Syntax.positions -- atomic parse trees are always annotated;
wenzelm
parents:
45666
diff
changeset
|
139 |
fun parsetree_to_ast ctxt raw trf parsetree = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
140 |
let |
44736 | 141 |
val reports = Unsynchronized.ref ([]: Position.report list); |
44735 | 142 |
fun report pos = Position.store_reports reports [pos]; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
143 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
144 |
fun trans a args = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
145 |
(case trf a of |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
146 |
NONE => Ast.mk_appl (Ast.Constant a) args |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
147 |
| SOME f => f ctxt args); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
148 |
|
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
149 |
fun asts_of_token tok = |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
150 |
if Lexicon.valued_token tok |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
151 |
then [Ast.Variable (Lexicon.str_of_token tok)] |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
152 |
else []; |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
153 |
|
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
154 |
fun asts_of_position c tok = |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
155 |
if raw then asts_of_token tok |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
156 |
else |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
157 |
[Ast.Appl [Ast.Constant c, ast_of (Parser.Tip tok), |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
158 |
Ast.Variable (Term_Position.encode (Lexicon.pos_of_token tok))]] |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
159 |
|
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
160 |
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
|
161 |
let |
42470 | 162 |
val pos = Lexicon.pos_of_token tok; |
163 |
val c = Proof_Context.read_class ctxt (Lexicon.str_of_token tok) |
|
48992 | 164 |
handle ERROR msg => error (msg ^ Position.here pos); |
42470 | 165 |
val _ = report pos (markup_class ctxt) c; |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
166 |
in [Ast.Constant (Lexicon.mark_class c)] end |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
167 |
| asts_of (Parser.Node ("_type_name", [Parser.Tip tok])) = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
168 |
let |
42470 | 169 |
val pos = Lexicon.pos_of_token tok; |
170 |
val Type (c, _) = |
|
171 |
Proof_Context.read_type_name_proper ctxt false (Lexicon.str_of_token tok) |
|
48992 | 172 |
handle ERROR msg => error (msg ^ Position.here pos); |
42470 | 173 |
val _ = report pos (markup_type ctxt) c; |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
174 |
in [Ast.Constant (Lexicon.mark_type c)] end |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
175 |
| 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
|
176 |
| asts_of (Parser.Node ("_position_sort", [Parser.Tip tok])) = asts_of_position "_ofsort" tok |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
177 |
| asts_of (Parser.Node (a, pts)) = |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
178 |
let |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
179 |
val _ = pts |> List.app |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
180 |
(fn Parser.Node _ => () | Parser.Tip tok => |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
181 |
if Lexicon.valued_token tok then () |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
182 |
else report (Lexicon.pos_of_token tok) (markup_entity ctxt) a); |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
183 |
in [trans a (maps asts_of pts)] end |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
184 |
| asts_of (Parser.Tip tok) = asts_of_token tok |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
185 |
|
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
186 |
and ast_of pt = |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
187 |
(case asts_of pt of |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
188 |
[ast] => ast |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
189 |
| 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
|
190 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
191 |
val ast = Exn.interruptible_capture ast_of parsetree; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
192 |
in (! reports, ast) end; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
193 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
194 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
195 |
(* ast_to_term *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
196 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
197 |
fun ast_to_term ctxt trf = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
198 |
let |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
199 |
fun trans a args = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
200 |
(case trf a of |
42476 | 201 |
NONE => Term.list_comb (Syntax.const a, args) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
202 |
| SOME f => f ctxt args); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
203 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
204 |
fun term_of (Ast.Constant a) = trans a [] |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
205 |
| term_of (Ast.Variable x) = Lexicon.read_var x |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
206 |
| term_of (Ast.Appl (Ast.Constant a :: (asts as _ :: _))) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
207 |
trans a (map term_of asts) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
208 |
| term_of (Ast.Appl (ast :: (asts as _ :: _))) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
209 |
Term.list_comb (term_of ast, map term_of asts) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
210 |
| 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
|
211 |
in term_of end; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
212 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
213 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
214 |
(* decode_term -- transform parse tree into raw term *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
215 |
|
44736 | 216 |
fun decode_term _ (result as (_: Position.report list, Exn.Exn _)) = result |
43761
e72ba84ae58f
tuned signature -- corresponding to Scala version;
wenzelm
parents:
43731
diff
changeset
|
217 |
| decode_term ctxt (reports0, Exn.Res tm) = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
218 |
let |
42250
cc5ac538f991
eliminated odd object-oriented type_context/term_context;
wenzelm
parents:
42249
diff
changeset
|
219 |
fun get_const a = |
42360 | 220 |
((true, #1 (Term.dest_Const (Proof_Context.read_const_proper ctxt false a))) |
221 |
handle ERROR _ => (false, Consts.intern (Proof_Context.consts_of ctxt) a)); |
|
222 |
val get_free = Proof_Context.intern_skolem ctxt; |
|
42250
cc5ac538f991
eliminated odd object-oriented type_context/term_context;
wenzelm
parents:
42249
diff
changeset
|
223 |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
224 |
val reports = Unsynchronized.ref reports0; |
44735 | 225 |
fun report ps = Position.store_reports reports ps; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
226 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
227 |
fun decode ps qs bs (Const ("_constrain", _) $ t $ typ) = |
42264 | 228 |
(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
|
229 |
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
|
230 |
| 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
|
231 |
| decode ps qs bs (Const ("_constrainAbs", _) $ t $ typ) = |
42264 | 232 |
(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
|
233 |
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
|
234 |
| 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
|
235 |
| decode _ qs bs (Abs (x, T, t)) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
236 |
let |
45412 | 237 |
val id = serial (); |
238 |
val _ = report qs (markup_bound true qs) (x, id); |
|
239 |
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
|
240 |
| decode _ _ bs (t $ u) = decode [] [] bs t $ decode [] [] bs u |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
241 |
| decode ps _ _ (Const (a, T)) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
242 |
(case try Lexicon.unmark_fixed a of |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
243 |
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
|
244 |
| NONE => |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
245 |
let |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
246 |
val c = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
247 |
(case try Lexicon.unmark_const a of |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
248 |
SOME c => c |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
249 |
| NONE => snd (get_const a)); |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
250 |
val _ = report ps (markup_const ctxt) c; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
251 |
in Const (c, T) end) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
252 |
| decode ps _ _ (Free (a, T)) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
253 |
(case (get_free a, get_const a) of |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
254 |
(SOME x, _) => (report ps (markup_free ctxt) x; Free (x, T)) |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
255 |
| (_, (true, c)) => (report ps (markup_const ctxt) c; Const (c, T)) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
256 |
| (_, (false, c)) => |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
257 |
if Long_Name.is_qualified c |
42282
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
258 |
then (report ps (markup_const ctxt) c; Const (c, T)) |
4fa41e068ff0
report literal tokens according to parsetree head;
wenzelm
parents:
42281
diff
changeset
|
259 |
else (report ps (markup_free ctxt) c; Free (c, T))) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
260 |
| 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
|
261 |
| decode ps _ bs (t as Bound i) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
262 |
(case try (nth bs) i of |
45412 | 263 |
SOME (qs, (x, id)) => (report ps (markup_bound false qs) (x, id); t) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
264 |
| NONE => t); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
265 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
266 |
val tm' = Exn.interruptible_capture (fn () => decode [] [] [] tm) (); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
267 |
in (! reports, tm') end; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
268 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
269 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
270 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
271 |
(** parse **) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
272 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
273 |
(* results *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
274 |
|
43761
e72ba84ae58f
tuned signature -- corresponding to Scala version;
wenzelm
parents:
43731
diff
changeset
|
275 |
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
|
276 |
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
|
277 |
|
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
278 |
fun report_result ctxt pos ambig_msgs results = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
279 |
(case (proper_results results, failed_results results) of |
44736 | 280 |
([], (reports, exn) :: _) => (Context_Position.reports ctxt reports; reraise exn) |
281 |
| ([(reports, x)], _) => (Context_Position.reports ctxt reports; x) |
|
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
282 |
| _ => |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
283 |
if null ambig_msgs then |
48992 | 284 |
error ("Parse error: ambiguous syntax" ^ Position.here pos) |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
285 |
else error (cat_lines ambig_msgs)); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
286 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
287 |
|
42249 | 288 |
(* parse raw asts *) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
289 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
290 |
fun parse_asts ctxt raw root (syms, pos) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
291 |
let |
42360 | 292 |
val syn = Proof_Context.syn_of ctxt; |
42253 | 293 |
val ast_tr = Syntax.parse_ast_translation syn; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
294 |
|
42251 | 295 |
val toks = Syntax.tokenize syn raw syms; |
44736 | 296 |
val _ = Context_Position.reports ctxt (map Lexicon.report_of_token toks); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
297 |
|
45641 | 298 |
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
|
299 |
handle ERROR msg => |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
300 |
error (msg ^ |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
301 |
implode (map (Markup.markup Markup.report o Lexicon.reported_token_range ctxt) toks)); |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
302 |
val len = length pts; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
303 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
304 |
val limit = Config.get ctxt Syntax.ambiguity_limit; |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
305 |
val ambig_msgs = |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
306 |
if len <= 1 then [] |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
307 |
else |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
308 |
[cat_lines |
48992 | 309 |
(("Ambiguous input" ^ Position.here (Position.reset_range pos) ^ |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
310 |
"\nproduces " ^ string_of_int len ^ " parse trees" ^ |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
311 |
(if len <= limit then "" else " (" ^ string_of_int limit ^ " displayed)") ^ ":") :: |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
312 |
map (Pretty.string_of o Parser.pretty_parsetree) (take limit pts))]; |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
313 |
|
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
314 |
in (ambig_msgs, map (parsetree_to_ast ctxt raw ast_tr) pts) end; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
315 |
|
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
316 |
fun parse_tree ctxt root input = |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
317 |
let |
42360 | 318 |
val syn = Proof_Context.syn_of ctxt; |
42253 | 319 |
val tr = Syntax.parse_translation syn; |
42255 | 320 |
val parse_rules = Syntax.parse_rules syn; |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
321 |
val (ambig_msgs, asts) = parse_asts ctxt false root input; |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
322 |
val results = |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
323 |
(map o apsnd o Exn.maps_result) |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
324 |
(Ast.normalize ctxt parse_rules #> Exn.interruptible_capture (ast_to_term ctxt tr)) asts; |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
325 |
in (ambig_msgs, results) end; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
326 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
327 |
|
42249 | 328 |
(* parse logical entities *) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
329 |
|
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
330 |
fun parse_failed ctxt pos msg kind = |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
331 |
cat_error msg ("Failed to parse " ^ kind ^ |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
332 |
Markup.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
|
333 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
334 |
fun parse_sort ctxt = |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
335 |
Syntax.parse_token ctxt Term_XML.Decode.sort Markup.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
|
336 |
(fn (syms, pos) => |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
337 |
parse_tree ctxt "sort" (syms, pos) |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
338 |
|> uncurry (report_result ctxt pos) |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
339 |
|> 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
|
340 |
|> 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
|
341 |
handle ERROR msg => parse_failed ctxt pos msg "sort"); |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
342 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
343 |
fun parse_typ ctxt = |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
344 |
Syntax.parse_token ctxt Term_XML.Decode.typ Markup.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
|
345 |
(fn (syms, pos) => |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
346 |
parse_tree ctxt "type" (syms, pos) |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
347 |
|> uncurry (report_result ctxt pos) |
45427
fca432074fb2
sort assignment before simultaneous term_check, not isolated parse_term;
wenzelm
parents:
45423
diff
changeset
|
348 |
|> 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
|
349 |
handle ERROR msg => parse_failed ctxt pos msg "type"); |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
350 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
351 |
fun parse_term is_prop ctxt = |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
352 |
let |
42281 | 353 |
val (markup, kind, root, constrain) = |
354 |
if is_prop |
|
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
355 |
then (Markup.prop, "proposition", "prop", Type.constraint propT) |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
356 |
else (Markup.term, "term", Config.get ctxt Syntax.root, I); |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
357 |
val decode = constrain o Term_XML.Decode.term; |
42249 | 358 |
in |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
359 |
Syntax.parse_token ctxt decode markup |
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
360 |
(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
|
361 |
let |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
362 |
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
|
363 |
val parsed_len = length (proper_results results); |
42249 | 364 |
|
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
365 |
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
|
366 |
val limit = Config.get ctxt Syntax.ambiguity_limit; |
42249 | 367 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
368 |
(*brute-force disambiguation via type-inference*) |
43761
e72ba84ae58f
tuned signature -- corresponding to Scala version;
wenzelm
parents:
43731
diff
changeset
|
369 |
fun check t = (Syntax.check_term ctxt (constrain t); Exn.Res t) |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
370 |
handle exn as ERROR _ => Exn.Exn exn; |
42249 | 371 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
372 |
val results' = |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
373 |
if parsed_len > 1 then |
46989 | 374 |
(grouped 10 (Par_List.map_name "Syntax_Phases.parse_term") o apsnd o Exn.maps_result) |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
375 |
check results |
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
376 |
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
|
377 |
val reports' = fst (hd results'); |
42249 | 378 |
|
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
379 |
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
|
380 |
val checked = map snd (proper_results results'); |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
381 |
val checked_len = length checked; |
42249 | 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 |
val show_term = Syntax.string_of_term (Config.put Printer.show_brackets true ctxt); |
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
384 |
in |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
385 |
if checked_len = 0 then |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
386 |
report_result ctxt pos [] |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
387 |
[(reports', Exn.Exn (Exn.EXCEPTIONS (map ERROR ambig_msgs @ errs)))] |
46506
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
388 |
else if checked_len = 1 then |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
389 |
(if parsed_len > 1 andalso ambiguity_warning then |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
390 |
Context_Position.if_visible ctxt warning |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
391 |
(cat_lines (ambig_msgs @ |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
392 |
["Fortunately, only one parse tree is type correct" ^ |
48992 | 393 |
Position.here (Position.reset_range pos) ^ |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
394 |
",\nbut you may still want to disambiguate your grammar or your input."])) |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
395 |
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
|
396 |
else |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
397 |
report_result ctxt pos [] |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
398 |
[(reports', Exn.Exn (ERROR (cat_lines (ambig_msgs @ |
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
399 |
(("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
|
400 |
(if checked_len <= limit then "" |
c7faa011bfa7
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46126
diff
changeset
|
401 |
else " (" ^ string_of_int limit ^ " displayed)") ^ ":") :: |
43731
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
402 |
map show_term (take limit checked))))))] |
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
wenzelm
parents:
43552
diff
changeset
|
403 |
end handle ERROR msg => parse_failed ctxt pos msg kind) |
42249 | 404 |
end; |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
405 |
|
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
406 |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
407 |
(* parse_ast_pattern *) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
408 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
409 |
fun parse_ast_pattern ctxt (root, str) = |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
410 |
let |
42360 | 411 |
val syn = Proof_Context.syn_of ctxt; |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
412 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
413 |
fun constify (ast as Ast.Constant _) = ast |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
414 |
| constify (ast as Ast.Variable x) = |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
415 |
if is_some (Syntax.lookup_const syn x) orelse Long_Name.is_qualified x |
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
416 |
then Ast.Constant x |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
417 |
else ast |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
418 |
| constify (Ast.Appl asts) = Ast.Appl (map constify asts); |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
419 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
420 |
val (syms, pos) = Syntax.read_token str; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
421 |
in |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
422 |
parse_asts ctxt true root (syms, pos) |
46512
4f9f61f9b535
simplified configuration options for syntax ambiguity;
wenzelm
parents:
46506
diff
changeset
|
423 |
|> uncurry (report_result ctxt pos) |
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
424 |
|> constify |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
425 |
end; |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
426 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
427 |
|
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
428 |
|
42245 | 429 |
(** encode parse trees **) |
430 |
||
431 |
(* term_of_sort *) |
|
432 |
||
433 |
fun term_of_sort S = |
|
434 |
let |
|
42476 | 435 |
val class = Syntax.const o Lexicon.mark_class; |
42245 | 436 |
|
437 |
fun classes [c] = class c |
|
42476 | 438 |
| classes (c :: cs) = Syntax.const "_classes" $ class c $ classes cs; |
42245 | 439 |
in |
440 |
(case S of |
|
42476 | 441 |
[] => Syntax.const "_topsort" |
42245 | 442 |
| [c] => class c |
42476 | 443 |
| cs => Syntax.const "_sort" $ classes cs) |
42245 | 444 |
end; |
445 |
||
446 |
||
447 |
(* term_of_typ *) |
|
448 |
||
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
449 |
fun term_of_typ ctxt ty = |
42245 | 450 |
let |
49690
a6814de45b69
more explicit show_type_constraint, show_sort_constraint;
wenzelm
parents:
49686
diff
changeset
|
451 |
val show_sort_constraint = Printer.show_sort_constraint ctxt; |
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
452 |
|
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
453 |
fun ofsort t raw_S = |
49690
a6814de45b69
more explicit show_type_constraint, show_sort_constraint;
wenzelm
parents:
49686
diff
changeset
|
454 |
if show_sort_constraint then |
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
455 |
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
|
456 |
in if S = dummyS then t else Syntax.const "_ofsort" $ t $ term_of_sort S end |
42245 | 457 |
else t; |
458 |
||
459 |
fun term_of (Type (a, Ts)) = |
|
42476 | 460 |
Term.list_comb (Syntax.const (Lexicon.mark_type a), map term_of Ts) |
42245 | 461 |
| term_of (TFree (x, S)) = |
42290
b1f544c84040
discontinued special treatment of structure Lexicon;
wenzelm
parents:
42289
diff
changeset
|
462 |
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
|
463 |
else ofsort (Syntax.const "_tfree" $ Syntax.free x) S |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
464 |
| term_of (TVar (xi, S)) = ofsort (Syntax.const "_tvar" $ Syntax.var xi) S; |
42245 | 465 |
in term_of ty end; |
466 |
||
467 |
||
468 |
(* simple_ast_of *) |
|
469 |
||
470 |
fun simple_ast_of ctxt = |
|
471 |
let |
|
472 |
val tune_var = if Config.get ctxt show_question_marks then I else unprefix "?"; |
|
473 |
fun ast_of (Const (c, _)) = Ast.Constant c |
|
474 |
| ast_of (Free (x, _)) = Ast.Variable x |
|
475 |
| ast_of (Var (xi, _)) = Ast.Variable (tune_var (Term.string_of_vname xi)) |
|
476 |
| ast_of (t as _ $ _) = |
|
477 |
let val (f, args) = strip_comb t |
|
478 |
in Ast.mk_appl (ast_of f) (map ast_of args) end |
|
42408 | 479 |
| ast_of (Bound i) = Ast.Appl [Ast.Constant "_loose", Ast.Variable ("B." ^ string_of_int i)] |
42245 | 480 |
| ast_of (Abs _) = raise Fail "simple_ast_of: Abs"; |
481 |
in ast_of end; |
|
482 |
||
483 |
||
484 |
(* sort_to_ast and typ_to_ast *) |
|
485 |
||
486 |
fun ast_of_termT ctxt trf tm = |
|
487 |
let |
|
488 |
val ctxt' = Config.put show_sorts false ctxt; |
|
489 |
fun ast_of (t as Const ("_tfree", _) $ Free _) = simple_ast_of ctxt t |
|
490 |
| ast_of (t as Const ("_tvar", _) $ Var _) = simple_ast_of ctxt t |
|
491 |
| ast_of (Const (a, _)) = trans a [] |
|
492 |
| ast_of (t as _ $ _) = |
|
493 |
(case strip_comb t of |
|
494 |
(Const (a, _), args) => trans a args |
|
495 |
| (f, args) => Ast.Appl (map ast_of (f :: args))) |
|
496 |
| ast_of t = simple_ast_of ctxt t |
|
42254 | 497 |
and trans a args = ast_of (trf a ctxt' dummyT args) |
498 |
handle Match => Ast.mk_appl (Ast.Constant a) (map ast_of args); |
|
42245 | 499 |
in ast_of tm end; |
500 |
||
501 |
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
|
502 |
fun typ_to_ast ctxt trf T = ast_of_termT ctxt trf (term_of_typ ctxt T); |
42245 | 503 |
|
504 |
||
505 |
(* term_to_ast *) |
|
506 |
||
42252 | 507 |
fun term_to_ast idents is_syntax_const ctxt trf tm = |
42245 | 508 |
let |
509 |
val show_types = |
|
510 |
Config.get ctxt show_types orelse Config.get ctxt show_sorts orelse |
|
511 |
Config.get ctxt show_all_types; |
|
512 |
val show_structs = Config.get ctxt show_structs; |
|
513 |
val show_free_types = Config.get ctxt show_free_types; |
|
514 |
val show_all_types = Config.get ctxt show_all_types; |
|
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
515 |
val show_markup = Config.get ctxt show_markup; |
42245 | 516 |
|
517 |
val {structs, fixes} = idents; |
|
518 |
||
42249 | 519 |
fun mark_atoms ((t as Const (c, _)) $ u) = |
42294 | 520 |
if member (op =) Syntax.token_markers c |
42245 | 521 |
then t $ u else mark_atoms t $ mark_atoms u |
522 |
| mark_atoms (t $ u) = mark_atoms t $ mark_atoms u |
|
523 |
| mark_atoms (Abs (x, T, t)) = Abs (x, T, mark_atoms t) |
|
524 |
| mark_atoms (t as Const (c, T)) = |
|
42252 | 525 |
if is_syntax_const c then t |
42245 | 526 |
else Const (Lexicon.mark_const c, T) |
527 |
| mark_atoms (t as Free (x, T)) = |
|
528 |
let val i = find_index (fn s => s = x) structs + 1 in |
|
529 |
if i = 0 andalso member (op =) fixes x then |
|
530 |
Const (Lexicon.mark_fixed x, T) |
|
531 |
else if i = 1 andalso not show_structs then |
|
42476 | 532 |
Syntax.const "_struct" $ Syntax.const "_indexdefault" |
533 |
else Syntax.const "_free" $ t |
|
42245 | 534 |
end |
535 |
| mark_atoms (t as Var (xi, T)) = |
|
42288
2074b31650e6
discontinued special treatment of structure Syntax_Ext (formerly Syn_Ext);
wenzelm
parents:
42284
diff
changeset
|
536 |
if xi = Syntax_Ext.dddot_indexname then Const ("_DDDOT", T) |
42476 | 537 |
else Syntax.const "_var" $ t |
42245 | 538 |
| mark_atoms a = a; |
539 |
||
540 |
fun prune_typs (t_seen as (Const _, _)) = t_seen |
|
541 |
| prune_typs (t as Free (x, ty), seen) = |
|
542 |
if ty = dummyT then (t, seen) |
|
42290
b1f544c84040
discontinued special treatment of structure Lexicon;
wenzelm
parents:
42289
diff
changeset
|
543 |
else if not show_free_types orelse member (op aconv) seen t then (Syntax.free x, seen) |
42245 | 544 |
else (t, t :: seen) |
545 |
| prune_typs (t as Var (xi, ty), seen) = |
|
546 |
if ty = dummyT then (t, seen) |
|
42290
b1f544c84040
discontinued special treatment of structure Lexicon;
wenzelm
parents:
42289
diff
changeset
|
547 |
else if not show_free_types orelse member (op aconv) seen t then (Syntax.var xi, seen) |
42245 | 548 |
else (t, t :: seen) |
549 |
| prune_typs (t_seen as (Bound _, _)) = t_seen |
|
550 |
| prune_typs (Abs (x, ty, t), seen) = |
|
551 |
let val (t', seen') = prune_typs (t, seen); |
|
552 |
in (Abs (x, ty, t'), seen') end |
|
553 |
| prune_typs (t1 $ t2, seen) = |
|
554 |
let |
|
555 |
val (t1', seen') = prune_typs (t1, seen); |
|
556 |
val (t2', seen'') = prune_typs (t2, seen'); |
|
557 |
in (t1' $ t2', seen'') end; |
|
558 |
||
559 |
fun ast_of tm = |
|
560 |
(case strip_comb tm of |
|
42284 | 561 |
(t as Abs _, ts) => Ast.mk_appl (ast_of (Syntax_Trans.abs_tr' ctxt t)) (map ast_of ts) |
42245 | 562 |
| ((c as Const ("_free", _)), Free (x, T) :: ts) => |
42290
b1f544c84040
discontinued special treatment of structure Lexicon;
wenzelm
parents:
42289
diff
changeset
|
563 |
Ast.mk_appl (constrain (c $ Syntax.free x) T) (map ast_of ts) |
42245 | 564 |
| ((c as Const ("_var", _)), Var (xi, T) :: ts) => |
42290
b1f544c84040
discontinued special treatment of structure Lexicon;
wenzelm
parents:
42289
diff
changeset
|
565 |
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
|
566 |
| ((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
|
567 |
let |
de49d9b4d7bc
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm
parents:
49659
diff
changeset
|
568 |
val X = |
de49d9b4d7bc
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm
parents:
49659
diff
changeset
|
569 |
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
|
570 |
else dummyT; |
de49d9b4d7bc
more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
wenzelm
parents:
49659
diff
changeset
|
571 |
in Ast.mk_appl (constrain (c $ Syntax.free x) X) (map ast_of ts) end |
42245 | 572 |
| (Const ("_idtdummy", T), ts) => |
42476 | 573 |
Ast.mk_appl (constrain (Syntax.const "_idtdummy") T) (map ast_of ts) |
42245 | 574 |
| (const as Const (c, T), ts) => |
575 |
if show_all_types |
|
576 |
then Ast.mk_appl (constrain const T) (map ast_of ts) |
|
577 |
else trans c T ts |
|
578 |
| (t, ts) => Ast.mk_appl (simple_ast_of ctxt t) (map ast_of ts)) |
|
579 |
||
42254 | 580 |
and trans a T args = ast_of (trf a ctxt T args) |
581 |
handle Match => Ast.mk_appl (Ast.Constant a) (map ast_of args) |
|
42245 | 582 |
|
583 |
and constrain t T = |
|
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
584 |
if (show_types orelse show_markup) andalso T <> dummyT then |
42248 | 585 |
Ast.Appl [Ast.Constant "_constrain", simple_ast_of ctxt t, |
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
586 |
ast_of_termT ctxt trf (term_of_typ ctxt T)] |
42245 | 587 |
else simple_ast_of ctxt t; |
588 |
in |
|
589 |
tm |
|
42284 | 590 |
|> Syntax_Trans.prop_tr' |
49659
251342b60a82
explicit show_types takes preferenced over show_markup;
wenzelm
parents:
49657
diff
changeset
|
591 |
|> show_types ? (#1 o prune_typs o rpair []) |
42245 | 592 |
|> mark_atoms |
593 |
|> ast_of |
|
594 |
end; |
|
595 |
||
596 |
||
597 |
||
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
598 |
(** unparse **) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
599 |
|
42245 | 600 |
local |
601 |
||
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
602 |
fun free_or_skolem ctxt x = |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
603 |
let |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
604 |
val m = |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
605 |
if Variable.is_fixed ctxt x orelse Syntax.is_pretty_global ctxt |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
606 |
then Markup.fixed x else Markup.intensify; |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
607 |
in |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
608 |
if can Name.dest_skolem x |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
609 |
then ([m, Markup.skolem], Variable.revert_fixed ctxt x) |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
610 |
else ([m, Markup.free], x) |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
611 |
end; |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
612 |
|
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
613 |
fun var_or_skolem s = |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
614 |
(case Lexicon.read_variable s of |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
615 |
SOME (x, i) => |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
616 |
(case try Name.dest_skolem x of |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
617 |
NONE => (Markup.var, s) |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
618 |
| SOME x' => (Markup.skolem, Term.string_of_vname (x', i))) |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
619 |
| NONE => (Markup.var, s)); |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
620 |
|
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
621 |
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
|
622 |
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
|
623 |
|
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
624 |
fun unparse_t t_to_ast prt_t markup ctxt t = |
42245 | 625 |
let |
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
626 |
val show_markup = Config.get ctxt show_markup; |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
627 |
val show_sorts = Config.get ctxt show_sorts; |
49659
251342b60a82
explicit show_types takes preferenced over show_markup;
wenzelm
parents:
49657
diff
changeset
|
628 |
val show_types = |
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
629 |
Config.get ctxt show_types orelse show_sorts orelse |
49659
251342b60a82
explicit show_types takes preferenced over show_markup;
wenzelm
parents:
49657
diff
changeset
|
630 |
Config.get ctxt show_all_types; |
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
631 |
|
42360 | 632 |
val syn = Proof_Context.syn_of ctxt; |
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
633 |
val prtabs = Syntax.prtabs syn; |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
634 |
val trf = Syntax.print_ast_translation syn; |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
635 |
|
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
636 |
fun markup_extern c = |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
637 |
(case Syntax.lookup_const syn c of |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
638 |
SOME "" => ([], c) |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
639 |
| SOME b => markup_extern b |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
640 |
| NONE => c |> Lexicon.unmark |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
641 |
{case_class = fn x => (markup_class ctxt x, Proof_Context.extern_class ctxt x), |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
642 |
case_type = fn x => (markup_type ctxt x, Proof_Context.extern_type ctxt x), |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
643 |
case_const = fn x => (markup_const ctxt x, Proof_Context.extern_const ctxt x), |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
644 |
case_fixed = fn x => free_or_skolem ctxt x, |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
645 |
case_default = fn x => ([], x)}); |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
646 |
|
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
647 |
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
|
648 |
| 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
|
649 |
| 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
|
650 |
| token_trans "_bound" x = SOME (Pretty.mark_str (Markup.bound, x)) |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
651 |
| 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
|
652 |
| 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
|
653 |
| 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
|
654 |
| 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
|
655 |
| token_trans _ _ = NONE; |
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
656 |
|
49655 | 657 |
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
|
658 |
| markup_trans "_constrain" [t, ty] = constrain_trans t ty |
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
659 |
| 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
|
660 |
| 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
|
661 |
| markup_trans _ _ = NONE |
49655 | 662 |
|
49662
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
663 |
and constrain_trans t ty = |
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
664 |
if show_markup andalso not show_types then |
49662
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
665 |
let |
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
666 |
val ((bg1, bg2), en) = typing_elem; |
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
667 |
val bg = bg1 ^ Pretty.symbolic_output (pretty_typ_ast Markup.empty ty) ^ bg2; |
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
668 |
in SOME (Pretty.raw_markup (bg, en) (0, [pretty_ast Markup.empty t])) end |
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
669 |
else NONE |
de6be6922c19
proper handling of constraints stemming from idtyp_ast_tr';
wenzelm
parents:
49660
diff
changeset
|
670 |
|
49686
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
671 |
and ofsort_trans ty s = |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
672 |
if show_markup andalso not show_sorts then |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
673 |
let |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
674 |
val ((bg1, bg2), en) = sorting_elem; |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
675 |
val bg = bg1 ^ Pretty.symbolic_output (pretty_typ_ast Markup.empty s) ^ bg2; |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
676 |
in SOME (Pretty.raw_markup (bg, en) (0, [pretty_typ_ast Markup.empty ty])) end |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
677 |
else NONE |
678aa92e921c
printed "_ofsort" is subject to show_markup as well;
wenzelm
parents:
49685
diff
changeset
|
678 |
|
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
679 |
and pretty_typ_ast m ast = ast |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
680 |
|> Printer.pretty_typ_ast ctxt prtabs trf markup_trans markup_extern |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
681 |
|> Pretty.markup m |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
682 |
|
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
683 |
and pretty_ast m ast = ast |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
684 |
|> prt_t ctxt prtabs trf markup_trans markup_extern |
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
685 |
|> Pretty.markup m; |
42245 | 686 |
in |
42255 | 687 |
t_to_ast ctxt (Syntax.print_translation syn) t |
688 |
|> Ast.normalize ctxt (Syntax.print_rules syn) |
|
49657
40e4feac2921
turn constraints into Isabelle_Markup.typing, depending on show_markup options;
wenzelm
parents:
49655
diff
changeset
|
689 |
|> pretty_ast markup |
42245 | 690 |
end; |
691 |
||
692 |
in |
|
693 |
||
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
694 |
val unparse_sort = unparse_t sort_to_ast Printer.pretty_typ_ast Markup.sort; |
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
695 |
val unparse_typ = unparse_t typ_to_ast Printer.pretty_typ_ast Markup.typ; |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
696 |
|
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
697 |
fun unparse_term ctxt = |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
698 |
let |
42360 | 699 |
val thy = Proof_Context.theory_of ctxt; |
700 |
val syn = Proof_Context.syn_of ctxt; |
|
701 |
val idents = Local_Syntax.idents_of (Proof_Context.syntax_of ctxt); |
|
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
702 |
in |
42298
d622145603ee
more accurate markup for syntax consts, notably binders which point back to the original logical entity;
wenzelm
parents:
42296
diff
changeset
|
703 |
unparse_t (term_to_ast idents (is_some o Syntax.lookup_const syn)) |
42267
9566078ad905
simplified printer context: uniform externing and static token translations;
wenzelm
parents:
42264
diff
changeset
|
704 |
(Printer.pretty_term_ast (not (Pure_Thy.old_appl_syntax thy))) |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
49690
diff
changeset
|
705 |
Markup.term ctxt |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
706 |
end; |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
707 |
|
42249 | 708 |
end; |
709 |
||
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
710 |
|
42245 | 711 |
|
712 |
(** translations **) |
|
713 |
||
714 |
(* type propositions *) |
|
715 |
||
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
716 |
fun type_prop_tr' ctxt T [Const ("\\<^const>Pure.sort_constraint", _)] = |
42476 | 717 |
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
|
718 |
| type_prop_tr' ctxt T [t] = |
42476 | 719 |
Syntax.const "_ofclass" $ term_of_typ ctxt T $ t |
42245 | 720 |
| type_prop_tr' _ T ts = raise TYPE ("type_prop_tr'", [T], ts); |
721 |
||
722 |
||
723 |
(* type reflection *) |
|
724 |
||
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
725 |
fun type_tr' ctxt (Type ("itself", [T])) ts = |
42476 | 726 |
Term.list_comb (Syntax.const "_TYPE" $ term_of_typ ctxt T, ts) |
42245 | 727 |
| type_tr' _ _ _ = raise Match; |
728 |
||
729 |
||
730 |
(* type constraints *) |
|
731 |
||
42247
12fe41a92cd5
typed_print_translation: discontinued show_sorts argument;
wenzelm
parents:
42245
diff
changeset
|
732 |
fun type_constraint_tr' ctxt (Type ("fun", [T, _])) (t :: ts) = |
42476 | 733 |
Term.list_comb (Syntax.const "_constrain" $ t $ term_of_typ ctxt T, ts) |
42245 | 734 |
| type_constraint_tr' _ _ _ = raise Match; |
735 |
||
736 |
||
42295
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
737 |
(* authentic syntax *) |
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
738 |
|
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
739 |
fun const_ast_tr intern ctxt [Ast.Variable c] = |
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
740 |
let |
42360 | 741 |
val Const (c', _) = Proof_Context.read_const_proper ctxt false c; |
42295
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
742 |
val d = if intern then Lexicon.mark_const c' else c; |
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
743 |
in Ast.Constant d end |
42470 | 744 |
| const_ast_tr intern ctxt [Ast.Appl [Ast.Constant "_constrain", x, T as Ast.Variable pos]] = |
745 |
(Ast.Appl [Ast.Constant "_constrain", const_ast_tr intern ctxt [x], T] |
|
746 |
handle ERROR msg => |
|
48992 | 747 |
error (msg ^ Position.here (the_default Position.none (Term_Position.decode pos)))) |
42295
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
748 |
| const_ast_tr _ _ asts = raise Ast.AST ("const_ast_tr", asts); |
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
749 |
|
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
750 |
|
42245 | 751 |
(* setup translations *) |
752 |
||
753 |
val _ = Context.>> (Context.map_theory |
|
42295
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
754 |
(Sign.add_advanced_trfuns |
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
755 |
([("_context_const", const_ast_tr true), |
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
756 |
("_context_xconst", const_ast_tr false)], [], [], []) #> |
8fdbb3b10beb
moved CONST syntax/translations to their proper place;
wenzelm
parents:
42294
diff
changeset
|
757 |
Sign.add_advanced_trfunsT |
42245 | 758 |
[("_type_prop", type_prop_tr'), |
759 |
("\\<^const>TYPE", type_tr'), |
|
760 |
("_type_constraint_", type_constraint_tr')])); |
|
761 |
||
762 |
||
763 |
||
42382
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
764 |
(** check/uncheck **) |
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
765 |
|
45429 | 766 |
(* context-sensitive (un)checking *) |
767 |
||
768 |
type key = int * bool; |
|
769 |
||
770 |
structure Checks = Generic_Data |
|
771 |
( |
|
772 |
type 'a check = 'a list -> Proof.context -> ('a list * Proof.context) option; |
|
773 |
type T = |
|
774 |
((key * ((string * typ check) * stamp) list) list * |
|
775 |
(key * ((string * term check) * stamp) list) list); |
|
776 |
val empty = ([], []); |
|
777 |
val extend = I; |
|
778 |
fun merge ((typ_checks1, term_checks1), (typ_checks2, term_checks2)) : T = |
|
779 |
(AList.join (op =) (K (Library.merge (eq_snd (op =)))) (typ_checks1, typ_checks2), |
|
780 |
AList.join (op =) (K (Library.merge (eq_snd (op =)))) (term_checks1, term_checks2)); |
|
781 |
); |
|
782 |
||
783 |
fun print_checks ctxt = |
|
784 |
let |
|
785 |
fun split_checks checks = |
|
786 |
List.partition (fn ((_, un), _) => not un) checks |
|
787 |
|> pairself (map (fn ((i, _), fs) => (i, map (fst o fst) fs)) |
|
788 |
#> sort (int_ord o pairself fst)); |
|
789 |
fun pretty_checks kind checks = |
|
790 |
checks |> map (fn (i, names) => Pretty.block |
|
791 |
[Pretty.str (kind ^ " (stage " ^ signed_string_of_int i ^ "):"), |
|
792 |
Pretty.brk 1, Pretty.strs names]); |
|
793 |
||
794 |
val (typs, terms) = Checks.get (Context.Proof ctxt); |
|
795 |
val (typ_checks, typ_unchecks) = split_checks typs; |
|
796 |
val (term_checks, term_unchecks) = split_checks terms; |
|
797 |
in |
|
798 |
pretty_checks "typ_checks" typ_checks @ |
|
799 |
pretty_checks "term_checks" term_checks @ |
|
800 |
pretty_checks "typ_unchecks" typ_unchecks @ |
|
801 |
pretty_checks "term_unchecks" term_unchecks |
|
802 |
end |> Pretty.chunks |> Pretty.writeln; |
|
803 |
||
804 |
||
805 |
local |
|
806 |
||
807 |
fun context_check which (key: key) name f = |
|
808 |
Checks.map (which (AList.map_default op = (key, []) (cons ((name, f), stamp ())))); |
|
809 |
||
810 |
fun simple_check eq f xs ctxt = |
|
811 |
let val xs' = f ctxt xs |
|
812 |
in if eq_list eq (xs, xs') then NONE else SOME (xs', ctxt) end; |
|
813 |
||
814 |
in |
|
815 |
||
45444 | 816 |
fun typ_check' stage = context_check apfst (stage, false); |
817 |
fun term_check' stage = context_check apsnd (stage, false); |
|
818 |
fun typ_uncheck' stage = context_check apfst (stage, true); |
|
819 |
fun term_uncheck' stage = context_check apsnd (stage, true); |
|
45429 | 820 |
|
45444 | 821 |
fun typ_check key name f = typ_check' key name (simple_check (op =) f); |
822 |
fun term_check key name f = term_check' key name (simple_check (op aconv) f); |
|
823 |
fun typ_uncheck key name f = typ_uncheck' key name (simple_check (op =) f); |
|
824 |
fun term_uncheck key name f = term_uncheck' key name (simple_check (op aconv) f); |
|
45429 | 825 |
|
826 |
end; |
|
827 |
||
828 |
||
829 |
local |
|
830 |
||
831 |
fun check_stage fs = perhaps_loop (perhaps_apply (map uncurry fs)); |
|
832 |
fun check_all fs = perhaps_apply (map check_stage fs); |
|
833 |
||
834 |
fun check which uncheck ctxt0 xs0 = |
|
835 |
let |
|
836 |
val funs = which (Checks.get (Context.Proof ctxt0)) |
|
837 |
|> map_filter (fn ((i, u), fs) => if uncheck = u then SOME (i, map (snd o fst) fs) else NONE) |
|
838 |
|> Library.sort (int_ord o pairself fst) |> map snd |
|
839 |
|> not uncheck ? map rev; |
|
840 |
in #1 (perhaps (check_all funs) (xs0, ctxt0)) end; |
|
841 |
||
842 |
val apply_typ_check = check fst false; |
|
843 |
val apply_term_check = check snd false; |
|
844 |
val apply_typ_uncheck = check fst true; |
|
845 |
val apply_term_uncheck = check snd true; |
|
846 |
||
847 |
in |
|
848 |
||
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
849 |
fun check_typs ctxt raw_tys = |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
850 |
let |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
851 |
val (sorting_report, tys) = Proof_Context.prepare_sortsT ctxt raw_tys; |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
852 |
val _ = Context_Position.if_visible ctxt Output.report sorting_report; |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
853 |
in |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
854 |
tys |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
855 |
|> apply_typ_check ctxt |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
856 |
|> Term_Sharing.typs (Proof_Context.theory_of ctxt) |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
857 |
end; |
45423
92f91f990165
tuned signature -- emphasize internal role of these operations;
wenzelm
parents:
45412
diff
changeset
|
858 |
|
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
859 |
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
|
860 |
let |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
861 |
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
|
862 |
val (ts, ps) = Type_Infer_Context.prepare_positions ctxt raw_ts'; |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
863 |
|
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
864 |
val tys = map (Logic.mk_type o snd) ps; |
45448
018f8959c7a6
more efficient prepare_sorts -- bypass encoded positions;
wenzelm
parents:
45447
diff
changeset
|
865 |
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
|
866 |
|> 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
|
867 |
|> chop (length ts); |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
868 |
val typing_report = |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
869 |
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
|
870 |
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
|
871 |
cons (Position.reported_text pos Markup.typing |
49674
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
872 |
(Syntax.string_of_typ ctxt (Logic.dest_type ty))) |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
873 |
else I) ps tys' [] |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
874 |
|> implode; |
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
875 |
|
dbadb4d03cbc
report sort assignment of visible type variables;
wenzelm
parents:
49662
diff
changeset
|
876 |
val _ = Context_Position.if_visible ctxt Output.report (sorting_report ^ typing_report); |
45445
41e641a870de
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
wenzelm
parents:
45444
diff
changeset
|
877 |
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
|
878 |
|
42382
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
879 |
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
|
880 |
|
45429 | 881 |
val uncheck_typs = apply_typ_uncheck; |
882 |
val uncheck_terms = apply_term_uncheck; |
|
883 |
||
884 |
end; |
|
885 |
||
886 |
||
887 |
(* standard phases *) |
|
888 |
||
889 |
val _ = Context.>> |
|
890 |
(typ_check 0 "standard" Proof_Context.standard_typ_check #> |
|
891 |
term_check 0 "standard" |
|
892 |
(fn ctxt => Type_Infer_Context.infer_types ctxt #> map (Proof_Context.expand_abbrevs ctxt)) #> |
|
893 |
term_check 100 "standard_finish" Proof_Context.standard_term_check_finish #> |
|
894 |
term_uncheck 0 "standard" Proof_Context.standard_term_uncheck); |
|
42382
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
895 |
|
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
896 |
|
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
897 |
|
42242
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
898 |
(** install operations **) |
39261908e12f
moved decode/parse operations to standard_syntax.ML;
wenzelm
parents:
42241
diff
changeset
|
899 |
|
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
900 |
val _ = Syntax.install_operations |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
901 |
{parse_sort = parse_sort, |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
902 |
parse_typ = parse_typ, |
42281 | 903 |
parse_term = parse_term false, |
904 |
parse_prop = parse_term true, |
|
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
905 |
unparse_sort = unparse_sort, |
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
906 |
unparse_typ = unparse_typ, |
42382
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
907 |
unparse_term = unparse_term, |
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
908 |
check_typs = check_typs, |
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
909 |
check_terms = check_terms, |
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
910 |
check_props = check_props, |
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
911 |
uncheck_typs = uncheck_typs, |
dcd983ee2c29
provide structure Syntax early (before structure Type), back-patch check/uncheck later;
wenzelm
parents:
42379
diff
changeset
|
912 |
uncheck_terms = uncheck_terms}; |
42241
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
913 |
|
dd8029f71e1c
separate module for standard implementation of inner syntax operations;
wenzelm
parents:
diff
changeset
|
914 |
end; |