author | wenzelm |
Sun, 18 Oct 2015 20:28:29 +0200 | |
changeset 61473 | 34d1913f0b20 |
parent 61471 | 9d4c08af61b8 |
child 61595 | 3591274c607e |
permissions | -rw-r--r-- |
24581 | 1 |
(* Title: Pure/ML/ml_context.ML |
24574 | 2 |
Author: Makarius |
3 |
||
4 |
ML context and antiquotations. |
|
5 |
*) |
|
6 |
||
7 |
signature ML_CONTEXT = |
|
8 |
sig |
|
9 |
val the_generic_context: unit -> Context.generic |
|
26432
095e448b95a0
renamed ML_Context.the_context to ML_Context.the_global_context;
wenzelm
parents:
26416
diff
changeset
|
10 |
val the_global_context: unit -> theory |
24574 | 11 |
val the_local_context: unit -> Proof.context |
39164
e7e12555e763
ML_Context.thm and ML_Context.thms no longer pervasive;
wenzelm
parents:
39140
diff
changeset
|
12 |
val thm: xstring -> thm |
e7e12555e763
ML_Context.thm and ML_Context.thms no longer pervasive;
wenzelm
parents:
39140
diff
changeset
|
13 |
val thms: xstring -> thm list |
26455 | 14 |
val exec: (unit -> unit) -> Context.generic -> Context.generic |
56070 | 15 |
val check_antiquotation: Proof.context -> xstring * Position.T -> string |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
16 |
val struct_name: Proof.context -> string |
59112 | 17 |
val variant: string -> Proof.context -> string * Proof.context |
56205 | 18 |
type decl = Proof.context -> string * string |
59112 | 19 |
val value_decl: string -> string -> Proof.context -> decl * Proof.context |
58011
bc6bced136e5
tuned signature -- moved type src to Token, without aliases;
wenzelm
parents:
57834
diff
changeset
|
20 |
val add_antiquotation: binding -> (Token.src -> Proof.context -> decl * Proof.context) -> |
56205 | 21 |
theory -> theory |
59917
9830c944670f
more uniform "verbose" option to print name space;
wenzelm
parents:
59127
diff
changeset
|
22 |
val print_antiquotations: bool -> Proof.context -> unit |
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
23 |
val eval: ML_Compiler.flags -> Position.T -> ML_Lex.token Antiquote.antiquote list -> unit |
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
24 |
val eval_file: ML_Compiler.flags -> Path.T -> unit |
59064 | 25 |
val eval_source: ML_Compiler.flags -> Input.source -> unit |
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
26 |
val eval_in: Proof.context option -> ML_Compiler.flags -> Position.T -> |
37198
3af985b10550
replaced ML_Lex.read_antiq by more concise ML_Lex.read, which includes full read/report with explicit position information;
wenzelm
parents:
36959
diff
changeset
|
27 |
ML_Lex.token Antiquote.antiquote list -> unit |
59064 | 28 |
val eval_source_in: Proof.context option -> ML_Compiler.flags -> Input.source -> unit |
58991
92b6f4e68c5a
more careful ML source positions, for improved PIDE markup;
wenzelm
parents:
58979
diff
changeset
|
29 |
val expression: Position.range -> string -> string -> string -> |
58978
e42da880c61e
more position information, e.g. relevant for errors in generated ML source;
wenzelm
parents:
58928
diff
changeset
|
30 |
ML_Lex.token Antiquote.antiquote list -> Context.generic -> Context.generic |
25204 | 31 |
end |
24574 | 32 |
|
33 |
structure ML_Context: ML_CONTEXT = |
|
34 |
struct |
|
35 |
||
26416
a66f86ef7bb9
added store_thms etc. (formerly in Thy/thm_database.ML);
wenzelm
parents:
26405
diff
changeset
|
36 |
(** implicit ML context **) |
24574 | 37 |
|
26416
a66f86ef7bb9
added store_thms etc. (formerly in Thy/thm_database.ML);
wenzelm
parents:
26405
diff
changeset
|
38 |
val the_generic_context = Context.the_thread_data; |
26432
095e448b95a0
renamed ML_Context.the_context to ML_Context.the_global_context;
wenzelm
parents:
26416
diff
changeset
|
39 |
val the_global_context = Context.theory_of o the_generic_context; |
24574 | 40 |
val the_local_context = Context.proof_of o the_generic_context; |
41 |
||
42360 | 42 |
fun thm name = Proof_Context.get_thm (the_local_context ()) name; |
43 |
fun thms name = Proof_Context.get_thms (the_local_context ()) name; |
|
39164
e7e12555e763
ML_Context.thm and ML_Context.thms no longer pervasive;
wenzelm
parents:
39140
diff
changeset
|
44 |
|
26455 | 45 |
fun exec (e: unit -> unit) context = |
46 |
(case Context.setmp_thread_data (SOME context) (fn () => (e (); Context.thread_data ())) () of |
|
47 |
SOME context' => context' |
|
48 |
| NONE => error "Missing context after execution"); |
|
26416
a66f86ef7bb9
added store_thms etc. (formerly in Thy/thm_database.ML);
wenzelm
parents:
26405
diff
changeset
|
49 |
|
a66f86ef7bb9
added store_thms etc. (formerly in Thy/thm_database.ML);
wenzelm
parents:
26405
diff
changeset
|
50 |
|
24574 | 51 |
|
52 |
(** ML antiquotations **) |
|
53 |
||
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
54 |
(* names for generated environment *) |
59112 | 55 |
|
56 |
structure Names = Proof_Data |
|
57 |
( |
|
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
58 |
type T = string * Name.context; |
59112 | 59 |
val init_names = ML_Syntax.reserved |> fold Name.declare ["ML_context", "ML_print_depth"]; |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
60 |
fun init _ = ("Isabelle0", init_names); |
59112 | 61 |
); |
62 |
||
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
63 |
fun struct_name ctxt = #1 (Names.get ctxt); |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
64 |
val struct_begin = (Names.map o apfst) (fn _ => "Isabelle" ^ serial_string ()); |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
65 |
|
59112 | 66 |
fun variant a ctxt = |
67 |
let |
|
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
68 |
val names = #2 (Names.get ctxt); |
59112 | 69 |
val (b, names') = Name.variant (Name.desymbolize (SOME false) a) names; |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
70 |
val ctxt' = (Names.map o apsnd) (K names') ctxt; |
59112 | 71 |
in (b, ctxt') end; |
72 |
||
73 |
||
74 |
(* decl *) |
|
75 |
||
76 |
type decl = Proof.context -> string * string; (*final context -> ML env, ML body*) |
|
77 |
||
78 |
fun value_decl a s ctxt = |
|
79 |
let |
|
80 |
val (b, ctxt') = variant a ctxt; |
|
81 |
val env = "val " ^ b ^ " = " ^ s ^ ";\n"; |
|
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
82 |
val body = struct_name ctxt ^ "." ^ b; |
59112 | 83 |
fun decl (_: Proof.context) = (env, body); |
84 |
in (decl, ctxt') end; |
|
85 |
||
86 |
||
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
87 |
(* theory data *) |
27343
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
88 |
|
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
89 |
structure Antiquotations = Theory_Data |
43560
d1650e3720fd
ML antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
42360
diff
changeset
|
90 |
( |
58011
bc6bced136e5
tuned signature -- moved type src to Token, without aliases;
wenzelm
parents:
57834
diff
changeset
|
91 |
type T = (Token.src -> Proof.context -> decl * Proof.context) Name_Space.table; |
50201
c26369c9eda6
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
wenzelm
parents:
48992
diff
changeset
|
92 |
val empty : T = Name_Space.empty_table Markup.ML_antiquotationN; |
43560
d1650e3720fd
ML antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
42360
diff
changeset
|
93 |
val extend = I; |
d1650e3720fd
ML antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
42360
diff
changeset
|
94 |
fun merge data : T = Name_Space.merge_tables data; |
d1650e3720fd
ML antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
42360
diff
changeset
|
95 |
); |
27343
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
96 |
|
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
97 |
val get_antiquotations = Antiquotations.get o Proof_Context.theory_of; |
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
98 |
|
56070 | 99 |
fun check_antiquotation ctxt = |
100 |
#1 o Name_Space.check (Context.Proof ctxt) (get_antiquotations ctxt); |
|
101 |
||
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
102 |
fun add_antiquotation name f thy = thy |
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
103 |
|> Antiquotations.map (Name_Space.define (Context.Theory thy) true (name, f) #> snd); |
55743 | 104 |
|
59917
9830c944670f
more uniform "verbose" option to print name space;
wenzelm
parents:
59127
diff
changeset
|
105 |
fun print_antiquotations verbose ctxt = |
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
106 |
Pretty.big_list "ML antiquotations:" |
59917
9830c944670f
more uniform "verbose" option to print name space;
wenzelm
parents:
59127
diff
changeset
|
107 |
(map (Pretty.mark_str o #1) (Name_Space.markup_table verbose ctxt (get_antiquotations ctxt))) |
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
108 |
|> Pretty.writeln; |
27343
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
109 |
|
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
110 |
fun apply_antiquotation src ctxt = |
58011
bc6bced136e5
tuned signature -- moved type src to Token, without aliases;
wenzelm
parents:
57834
diff
changeset
|
111 |
let val (src', f) = Token.check_src ctxt (get_antiquotations ctxt) src |
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
112 |
in f src' ctxt end; |
43563 | 113 |
|
24574 | 114 |
|
27343
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
115 |
(* parsing and evaluation *) |
24574 | 116 |
|
27343
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
117 |
local |
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
118 |
|
24574 | 119 |
val antiq = |
56201 | 120 |
Parse.!!! (Parse.position Parse.xname -- Parse.args --| Scan.ahead Parse.eof) |
58011
bc6bced136e5
tuned signature -- moved type src to Token, without aliases;
wenzelm
parents:
57834
diff
changeset
|
121 |
>> uncurry Token.src; |
24574 | 122 |
|
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
123 |
fun make_env name visible = |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
124 |
(ML_Lex.tokenize |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
125 |
("structure " ^ name ^ " =\nstruct\n\ |
52663
6e71d43775e5
retain compile-time context visibility, which is particularly important for "apply tactic";
wenzelm
parents:
50201
diff
changeset
|
126 |
\val ML_context = Context_Position.set_visible " ^ Bool.toString visible ^ |
57832 | 127 |
" (ML_Context.the_local_context ());\n\ |
57834
0d295e339f52
prefer dynamic ML_print_depth if context happens to be available;
wenzelm
parents:
57832
diff
changeset
|
128 |
\val ML_print_depth =\n\ |
0d295e339f52
prefer dynamic ML_print_depth if context happens to be available;
wenzelm
parents:
57832
diff
changeset
|
129 |
\ let val default = ML_Options.get_print_depth ()\n\ |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
130 |
\ in fn () => ML_Options.get_print_depth_default default end;\n"), |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
131 |
ML_Lex.tokenize "end;"); |
48776
37cd53e69840
faster compilation of ML with antiquotations: static ML_context is bound once in auxiliary structure Isabelle;
wenzelm
parents:
47005
diff
changeset
|
132 |
|
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
133 |
fun reset_env name = ML_Lex.tokenize ("structure " ^ name ^ " = struct end"); |
28270
7ada24ebea94
explicit handling of ML environment within generic context;
wenzelm
parents:
27895
diff
changeset
|
134 |
|
59112 | 135 |
fun expanding (Antiquote.Text tok) = ML_Lex.is_cartouche tok |
61471 | 136 |
| expanding (Antiquote.Control _) = true |
59112 | 137 |
| expanding (Antiquote.Antiq _) = true; |
138 |
||
30637
3e3c2cd88cf1
export eval_antiquotes: refined version that operates on ML tokens;
wenzelm
parents:
30614
diff
changeset
|
139 |
fun eval_antiquotes (ants, pos) opt_context = |
24574 | 140 |
let |
52663
6e71d43775e5
retain compile-time context visibility, which is particularly important for "apply tactic";
wenzelm
parents:
50201
diff
changeset
|
141 |
val visible = |
6e71d43775e5
retain compile-time context visibility, which is particularly important for "apply tactic";
wenzelm
parents:
50201
diff
changeset
|
142 |
(case opt_context of |
6e71d43775e5
retain compile-time context visibility, which is particularly important for "apply tactic";
wenzelm
parents:
50201
diff
changeset
|
143 |
SOME (Context.Proof ctxt) => Context_Position.is_visible ctxt |
6e71d43775e5
retain compile-time context visibility, which is particularly important for "apply tactic";
wenzelm
parents:
50201
diff
changeset
|
144 |
| _ => true); |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
145 |
val opt_ctxt = Option.map Context.proof_of opt_context; |
52663
6e71d43775e5
retain compile-time context visibility, which is particularly important for "apply tactic";
wenzelm
parents:
50201
diff
changeset
|
146 |
|
27343
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
147 |
val ((ml_env, ml_body), opt_ctxt') = |
59112 | 148 |
if forall (not o expanding) ants |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
149 |
then (([], map (fn Antiquote.Text tok => tok) ants), opt_ctxt) |
27343
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
150 |
else |
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
151 |
let |
59112 | 152 |
fun tokenize range = apply2 (ML_Lex.tokenize #> map (ML_Lex.set_range range)); |
53167 | 153 |
|
61471 | 154 |
fun expand_src range src ctxt = |
155 |
let val (decl, ctxt') = apply_antiquotation src ctxt |
|
156 |
in (decl #> tokenize range, ctxt') end; |
|
157 |
||
158 |
fun expand (Antiquote.Text tok) ctxt = |
|
59112 | 159 |
if ML_Lex.is_cartouche tok then |
160 |
let |
|
161 |
val range = ML_Lex.range_of tok; |
|
162 |
val text = |
|
163 |
Symbol_Pos.explode (ML_Lex.content_of tok, #1 range) |
|
164 |
|> Symbol_Pos.cartouche_content |
|
165 |
|> Symbol_Pos.implode_range range |> #1; |
|
166 |
val (decl, ctxt') = |
|
167 |
value_decl "input" |
|
168 |
("Input.source true " ^ ML_Syntax.print_string text ^ " " ^ |
|
169 |
ML_Syntax.atomic (ML_Syntax.print_range range)) ctxt; |
|
170 |
in (decl #> tokenize range, ctxt') end |
|
61471 | 171 |
else (K ([], [tok]), ctxt) |
61473
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61471
diff
changeset
|
172 |
| expand (Antiquote.Control {name, range, body}) ctxt = |
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61471
diff
changeset
|
173 |
expand_src range (Token.src name [Token.read_cartouche body]) ctxt |
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61471
diff
changeset
|
174 |
| expand (Antiquote.Antiq {range, body, ...}) ctxt = |
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61471
diff
changeset
|
175 |
expand_src range |
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61471
diff
changeset
|
176 |
(Token.read_antiq (Thy_Header.get_keywords' ctxt) antiq (body, #1 range)) ctxt; |
53167 | 177 |
|
27343
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
178 |
val ctxt = |
4b28b80dd1f8
add_antiq: more general notion of ML antiquotation;
wenzelm
parents:
26881
diff
changeset
|
179 |
(case opt_ctxt of |
48992 | 180 |
NONE => error ("No context -- cannot expand ML antiquotations" ^ Position.here pos) |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
181 |
| SOME ctxt => struct_begin ctxt); |
27378 | 182 |
|
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
183 |
val (begin_env, end_env) = make_env (struct_name ctxt) visible; |
53167 | 184 |
val (decls, ctxt') = fold_map expand ants ctxt; |
52663
6e71d43775e5
retain compile-time context visibility, which is particularly important for "apply tactic";
wenzelm
parents:
50201
diff
changeset
|
185 |
val (ml_env, ml_body) = |
59058
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58991
diff
changeset
|
186 |
decls |> map (fn decl => decl ctxt') |> split_list |> apply2 flat; |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
187 |
in ((begin_env @ ml_env @ end_env, ml_body), SOME ctxt') end; |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
188 |
in ((ml_env, ml_body), opt_ctxt') end; |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
189 |
|
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
190 |
in |
24574 | 191 |
|
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
192 |
fun eval flags pos ants = |
24574 | 193 |
let |
56304
40274e4f5ebf
redirect ML_Compiler reports more directly: only the (big) parse tree report is deferred via Execution.print (NB: this does not work for asynchronous "diag" commands);
wenzelm
parents:
56303
diff
changeset
|
194 |
val non_verbose = ML_Compiler.verbose false flags; |
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
195 |
|
28270
7ada24ebea94
explicit handling of ML environment within generic context;
wenzelm
parents:
27895
diff
changeset
|
196 |
(*prepare source text*) |
41485
6c0de045d127
ML_trace: observe context visibility flag (import for Latex mode, for example);
wenzelm
parents:
41375
diff
changeset
|
197 |
val ((env, body), env_ctxt) = eval_antiquotes (ants, pos) (Context.thread_data ()); |
31334 | 198 |
val _ = |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
199 |
(case env_ctxt of |
41485
6c0de045d127
ML_trace: observe context visibility flag (import for Latex mode, for example);
wenzelm
parents:
41375
diff
changeset
|
200 |
SOME ctxt => |
56303
4cc3f4db3447
clarified Isabelle/ML bootstrap, such that Execution does not require ML_Compiler;
wenzelm
parents:
56294
diff
changeset
|
201 |
if Config.get ctxt ML_Options.source_trace andalso Context_Position.is_visible ctxt |
56294
85911b8a6868
prefer Context_Position where a context is available;
wenzelm
parents:
56279
diff
changeset
|
202 |
then tracing (cat_lines [ML_Lex.flatten env, ML_Lex.flatten body]) |
41375 | 203 |
else () |
204 |
| NONE => ()); |
|
28270
7ada24ebea94
explicit handling of ML environment within generic context;
wenzelm
parents:
27895
diff
changeset
|
205 |
|
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
206 |
(*prepare environment*) |
41485
6c0de045d127
ML_trace: observe context visibility flag (import for Latex mode, for example);
wenzelm
parents:
41375
diff
changeset
|
207 |
val _ = |
6c0de045d127
ML_trace: observe context visibility flag (import for Latex mode, for example);
wenzelm
parents:
41375
diff
changeset
|
208 |
Context.setmp_thread_data |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
209 |
(Option.map (Context.Proof o Context_Position.set_visible false) env_ctxt) |
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
210 |
(fn () => (ML_Compiler.eval non_verbose Position.none env; Context.thread_data ())) () |
31325
700951b53d21
moved local ML environment to separate module ML_Env;
wenzelm
parents:
30683
diff
changeset
|
211 |
|> (fn NONE => () | SOME context' => Context.>> (ML_Env.inherit context')); |
28270
7ada24ebea94
explicit handling of ML environment within generic context;
wenzelm
parents:
27895
diff
changeset
|
212 |
|
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
213 |
(*eval body*) |
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
214 |
val _ = ML_Compiler.eval flags pos body; |
59127
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
215 |
|
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
216 |
(*clear environment*) |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
217 |
val _ = |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
218 |
(case (env_ctxt, is_some (Context.thread_data ())) of |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
219 |
(SOME ctxt, true) => |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
220 |
let |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
221 |
val name = struct_name ctxt; |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
222 |
val _ = ML_Compiler.eval non_verbose Position.none (reset_env name); |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
223 |
val _ = Context.>> (ML_Env.forget_structure name); |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
224 |
in () end |
723b11f8ffbf
more careful handling of auxiliary environment structure -- allow nested ML evaluation;
wenzelm
parents:
59112
diff
changeset
|
225 |
| _ => ()); |
28270
7ada24ebea94
explicit handling of ML environment within generic context;
wenzelm
parents:
27895
diff
changeset
|
226 |
in () end; |
24574 | 227 |
|
228 |
end; |
|
229 |
||
230 |
||
30672
beaadd5af500
more systematic type use_context, with particular values ML_Parse.global_context and ML_Context.local_context;
wenzelm
parents:
30643
diff
changeset
|
231 |
(* derived versions *) |
24574 | 232 |
|
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
233 |
fun eval_file flags path = |
56203
76c72f4d0667
clarified bootstrap process: switch to ML with context and antiquotations earlier;
wenzelm
parents:
56201
diff
changeset
|
234 |
let val pos = Path.position path |
59067 | 235 |
in eval flags pos (ML_Lex.read_pos pos (File.read path)) end; |
56203
76c72f4d0667
clarified bootstrap process: switch to ML with context and antiquotations earlier;
wenzelm
parents:
56201
diff
changeset
|
236 |
|
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
237 |
fun eval_source flags source = |
59064 | 238 |
eval flags (Input.pos_of source) (ML_Lex.read_source (#SML flags) source); |
37198
3af985b10550
replaced ML_Lex.read_antiq by more concise ML_Lex.read, which includes full read/report with explicit position information;
wenzelm
parents:
36959
diff
changeset
|
239 |
|
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
240 |
fun eval_in ctxt flags pos ants = |
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
241 |
Context.setmp_thread_data (Option.map Context.Proof ctxt) |
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
242 |
(fn () => eval flags pos ants) (); |
24574 | 243 |
|
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
244 |
fun eval_source_in ctxt flags source = |
56069
451d5b73f8cf
simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
wenzelm
parents:
56032
diff
changeset
|
245 |
Context.setmp_thread_data (Option.map Context.Proof ctxt) |
56275
600f432ab556
added command 'SML_file' for Standard ML without Isabelle/ML add-ons;
wenzelm
parents:
56229
diff
changeset
|
246 |
(fn () => eval_source flags source) (); |
37198
3af985b10550
replaced ML_Lex.read_antiq by more concise ML_Lex.read, which includes full read/report with explicit position information;
wenzelm
parents:
36959
diff
changeset
|
247 |
|
58991
92b6f4e68c5a
more careful ML source positions, for improved PIDE markup;
wenzelm
parents:
58979
diff
changeset
|
248 |
fun expression range name constraint body ants = |
59067 | 249 |
exec (fn () => |
250 |
eval ML_Compiler.flags (#1 range) |
|
251 |
(ML_Lex.read "Context.set_thread_data (SOME (let val " @ ML_Lex.read_set_range range name @ |
|
252 |
ML_Lex.read (": " ^ constraint ^ " =") @ ants @ |
|
253 |
ML_Lex.read ("in " ^ body ^ " end (ML_Context.the_generic_context ())));"))); |
|
37198
3af985b10550
replaced ML_Lex.read_antiq by more concise ML_Lex.read, which includes full read/report with explicit position information;
wenzelm
parents:
36959
diff
changeset
|
254 |
|
24574 | 255 |
end; |
256 |