| author | wenzelm | 
| Sat, 29 Apr 2017 11:06:39 +0200 | |
| changeset 65633 | 826311fca263 | 
| parent 64959 | 9ca021bd718d | 
| child 66586 | e5e56c330976 | 
| permissions | -rw-r--r-- | 
| 37745 
6315b6426200
checking generated code for various target languages
 haftmann parents: 
37528diff
changeset | 1 | (* Title: Tools/Code/code_target.ML | 
| 24219 | 2 | Author: Florian Haftmann, TU Muenchen | 
| 3 | ||
| 38910 | 4 | Generic infrastructure for target language data. | 
| 24219 | 5 | *) | 
| 6 | ||
| 7 | signature CODE_TARGET = | |
| 8 | sig | |
| 55757 | 9 | val cert_tyco: Proof.context -> string -> string | 
| 10 | val read_tyco: Proof.context -> string -> string | |
| 36471 | 11 | |
| 55757 | 12 | val export_code_for: Proof.context -> Path.T option -> string -> int option -> string -> Token.T list | 
| 55683 | 13 | -> Code_Thingol.program -> bool -> Code_Symbol.T list -> unit | 
| 55757 | 14 | val produce_code_for: Proof.context -> string -> int option -> string -> Token.T list | 
| 55683 | 15 | -> Code_Thingol.program -> bool -> Code_Symbol.T list -> (string * string) list * string option list | 
| 55757 | 16 | val present_code_for: Proof.context -> string -> int option -> string -> Token.T list | 
| 55150 | 17 | -> Code_Thingol.program -> Code_Symbol.T list * Code_Symbol.T list -> string | 
| 55757 | 18 | val check_code_for: Proof.context -> string -> bool -> Token.T list | 
| 55683 | 19 | -> Code_Thingol.program -> bool -> Code_Symbol.T list -> unit | 
| 38918 | 20 | |
| 55757 | 21 | val export_code: Proof.context -> bool -> string list | 
| 38933 
bd77e092f67c
avoid strange special treatment of empty module names
 haftmann parents: 
38929diff
changeset | 22 | -> (((string * string) * Path.T option) * Token.T list) list -> unit | 
| 55757 | 23 | val produce_code: Proof.context -> bool -> string list | 
| 48568 | 24 | -> string -> int option -> string -> Token.T list -> (string * string) list * string option list | 
| 55757 | 25 | val present_code: Proof.context -> string list -> Code_Symbol.T list | 
| 38933 
bd77e092f67c
avoid strange special treatment of empty module names
 haftmann parents: 
38929diff
changeset | 26 | -> string -> int option -> string -> Token.T list -> string | 
| 55757 | 27 | val check_code: Proof.context -> bool -> string list | 
| 38918 | 28 | -> ((string * bool) * Token.T list) list -> unit | 
| 29 | ||
| 48568 | 30 | val generatedN: string | 
| 64957 | 31 | val compilation_text: Proof.context -> string -> Code_Thingol.program | 
| 55684 
ee49b4f7edc8
keep only identifiers public which are explicitly requested or demanded by dependencies
 haftmann parents: 
55683diff
changeset | 32 | -> Code_Symbol.T list -> bool -> ((string * class list) list * Code_Thingol.itype) * Code_Thingol.iterm | 
| 48568 | 33 | -> (string * string) list * string | 
| 64959 | 34 | val compilation_text': Proof.context -> string -> string option -> Code_Thingol.program | 
| 35 | -> Code_Symbol.T list -> bool -> ((string * class list) list * Code_Thingol.itype) * Code_Thingol.iterm | |
| 36 | -> ((string * string) list * string) * (Code_Symbol.T -> string option) | |
| 41344 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 37 | |
| 28054 | 38 | type serializer | 
| 34152 | 39 | type literals = Code_Printer.literals | 
| 59104 | 40 | type language | 
| 41 | type ancestry | |
| 59479 | 42 | val assert_target: theory -> string -> string | 
| 59104 | 43 | val add_language: string * language -> theory -> theory | 
| 44 | val add_derived_target: string * ancestry -> theory -> theory | |
| 55757 | 45 | val the_literals: Proof.context -> string -> literals | 
| 28054 | 46 | type serialization | 
| 36959 
f5417836dbea
renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
 wenzelm parents: 
36537diff
changeset | 47 | val parse_args: 'a parser -> Token.T list -> 'a | 
| 38916 | 48 | val serialization: (int -> Path.T option -> 'a -> unit) | 
| 55150 | 49 | -> (Code_Symbol.T list -> int -> 'a -> (string * string) list * (Code_Symbol.T -> string option)) | 
| 38925 | 50 | -> 'a -> serialization | 
| 59324 | 51 | val default_code_width: int Config.T | 
| 38917 | 52 | |
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 53 |   type ('a, 'b, 'c, 'd, 'e, 'f) symbol_attr_decl
 | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 54 | val set_identifiers: (string, string, string, string, string, string) symbol_attr_decl | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 55 | -> theory -> theory | 
| 55372 | 56 | val set_printings: (Code_Printer.raw_const_syntax, Code_Printer.tyco_syntax, string, unit, unit, (string * string list)) symbol_attr_decl | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 57 | -> theory -> theory | 
| 28054 | 58 | val add_reserved: string -> string -> theory -> theory | 
| 24219 | 59 | end; | 
| 60 | ||
| 28054 | 61 | structure Code_Target : CODE_TARGET = | 
| 24219 | 62 | struct | 
| 63 | ||
| 55150 | 64 | open Basic_Code_Symbol; | 
| 28054 | 65 | open Basic_Code_Thingol; | 
| 34152 | 66 | |
| 67 | type literals = Code_Printer.literals; | |
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 68 | type ('a, 'b, 'c, 'd, 'e, 'f) symbol_attr_decl =
 | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 69 | (string * (string * 'a option) list, string * (string * 'b option) list, | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 70 | class * (string * 'c option) list, (class * class) * (string * 'd option) list, | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 71 | (class * string) * (string * 'e option) list, | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 72 | string * (string * 'f option) list) Code_Symbol.attr; | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 73 | |
| 34152 | 74 | type tyco_syntax = Code_Printer.tyco_syntax; | 
| 55153 
eedd549de3ef
more suitable names, without any notion of "activating"
 haftmann parents: 
55150diff
changeset | 75 | type raw_const_syntax = Code_Printer.raw_const_syntax; | 
| 34152 | 76 | |
| 24219 | 77 | |
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 78 | (** checking and parsing of symbols **) | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 79 | |
| 55757 | 80 | fun cert_const ctxt const = | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 81 | let | 
| 55757 | 82 | val _ = if Sign.declared_const (Proof_Context.theory_of ctxt) const then () | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 83 |       else error ("No such constant: " ^ quote const);
 | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 84 | in const end; | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 85 | |
| 55757 | 86 | fun read_const ctxt = Code.read_const (Proof_Context.theory_of ctxt); | 
| 87 | ||
| 88 | fun cert_tyco ctxt tyco = | |
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 89 | let | 
| 55757 | 90 | val _ = if Sign.declared_tyname (Proof_Context.theory_of ctxt) tyco then () | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 91 |       else error ("No such type constructor: " ^ quote tyco);
 | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 92 | in tyco end; | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 93 | |
| 55951 
c07d184aebe9
tuned signature -- more uniform check_type_name/read_type_name;
 wenzelm parents: 
55776diff
changeset | 94 | fun read_tyco ctxt = | 
| 56002 | 95 |   #1 o dest_Type o Proof_Context.read_type_name {proper = true, strict = true} ctxt;
 | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 96 | |
| 55757 | 97 | fun cert_class ctxt class = | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 98 | let | 
| 55757 | 99 | val _ = Axclass.get_info (Proof_Context.theory_of ctxt) class; | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 100 | in class end; | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 101 | |
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 102 | val parse_classrel_ident = Parse.class --| @{keyword "<"} -- Parse.class;
 | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 103 | |
| 55757 | 104 | fun cert_inst ctxt (class, tyco) = | 
| 105 | (cert_class ctxt class, cert_tyco ctxt tyco); | |
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 106 | |
| 55757 | 107 | fun read_inst ctxt (raw_tyco, raw_class) = | 
| 108 | (read_tyco ctxt raw_tyco, Proof_Context.read_class ctxt raw_class); | |
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 109 | |
| 62969 | 110 | val parse_inst_ident = Parse.name --| @{keyword "::"} -- Parse.class;
 | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 111 | |
| 55757 | 112 | fun cert_syms ctxt = | 
| 113 | Code_Symbol.map_attr (apfst (cert_const ctxt)) (apfst (cert_tyco ctxt)) | |
| 59058 
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
 wenzelm parents: 
58928diff
changeset | 114 | (apfst (cert_class ctxt)) ((apfst o apply2) (cert_class ctxt)) (apfst (cert_inst ctxt)) I; | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 115 | |
| 55757 | 116 | fun read_syms ctxt = | 
| 117 | Code_Symbol.map_attr (apfst (read_const ctxt)) (apfst (read_tyco ctxt)) | |
| 59058 
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
 wenzelm parents: 
58928diff
changeset | 118 | (apfst (Proof_Context.read_class ctxt)) ((apfst o apply2) (Proof_Context.read_class ctxt)) (apfst (read_inst ctxt)) I; | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 119 | |
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 120 | fun check_name is_module s = | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 121 | let | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 122 | val _ = if s = "" then error "Bad empty code name" else (); | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 123 | val xs = Long_Name.explode s; | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 124 | val xs' = if is_module | 
| 56826 
ba18bd41e510
enforce case of identifiers only to accomodate strict language requirements (or clear separation of constructors from variables in the case of SML)
 haftmann parents: 
56811diff
changeset | 125 | then map (Name.desymbolize NONE) xs | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 126 | else if length xs < 2 | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 127 |         then error ("Bad code name without module component: " ^ quote s)
 | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 128 | else | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 129 | let | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 130 | val (ys, y) = split_last xs; | 
| 56826 
ba18bd41e510
enforce case of identifiers only to accomodate strict language requirements (or clear separation of constructors from variables in the case of SML)
 haftmann parents: 
56811diff
changeset | 131 | val ys' = map (Name.desymbolize NONE) ys; | 
| 
ba18bd41e510
enforce case of identifiers only to accomodate strict language requirements (or clear separation of constructors from variables in the case of SML)
 haftmann parents: 
56811diff
changeset | 132 | val y' = Name.desymbolize NONE y; | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 133 | in ys' @ [y'] end; | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 134 | in if xs' = xs | 
| 55291 | 135 | then if is_module then (xs, "") else split_last xs | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 136 |     else error ("Invalid code name: " ^ quote s ^ "\n"
 | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 137 | ^ "better try " ^ quote (Long_Name.implode xs')) | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 138 | end; | 
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 139 | |
| 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 140 | |
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 141 | (** serializations and serializer **) | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 142 | |
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 143 | (* serialization: abstract nonsense to cover different destinies for generated code *) | 
| 24219 | 144 | |
| 55150 | 145 | datatype destination = Export of Path.T option | Produce | Present of Code_Symbol.T list; | 
| 146 | type serialization = int -> destination -> ((string * string) list * (Code_Symbol.T -> string option)) option; | |
| 27014 
a5f53d9d2b60
yet another attempt to circumvent printmode problems
 haftmann parents: 
27001diff
changeset | 147 | |
| 39659 | 148 | fun serialization output _ content width (Export some_path) = | 
| 39661 
6381d18507ef
reverted cs 07549694e2f1 -- use re-printing with current print mode instead after code assembly, avoid Latex.output_typewriter
 haftmann parents: 
39659diff
changeset | 149 | (output width some_path content; NONE) | 
| 
6381d18507ef
reverted cs 07549694e2f1 -- use re-printing with current print mode instead after code assembly, avoid Latex.output_typewriter
 haftmann parents: 
39659diff
changeset | 150 | | serialization _ string content width Produce = | 
| 
6381d18507ef
reverted cs 07549694e2f1 -- use re-printing with current print mode instead after code assembly, avoid Latex.output_typewriter
 haftmann parents: 
39659diff
changeset | 151 | string [] width content |> SOME | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 152 | | serialization _ string content width (Present syms) = | 
| 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 153 | string syms width content | 
| 59430 | 154 | |> (apfst o map o apsnd) Output.output | 
| 39661 
6381d18507ef
reverted cs 07549694e2f1 -- use re-printing with current print mode instead after code assembly, avoid Latex.output_typewriter
 haftmann parents: 
39659diff
changeset | 155 | |> SOME; | 
| 39659 | 156 | |
| 39661 
6381d18507ef
reverted cs 07549694e2f1 -- use re-printing with current print mode instead after code assembly, avoid Latex.output_typewriter
 haftmann parents: 
39659diff
changeset | 157 | fun export some_path f = (f (Export some_path); ()); | 
| 
6381d18507ef
reverted cs 07549694e2f1 -- use re-printing with current print mode instead after code assembly, avoid Latex.output_typewriter
 haftmann parents: 
39659diff
changeset | 158 | fun produce f = the (f Produce); | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 159 | fun present syms f = space_implode "\n\n" (map snd (fst (the (f (Present syms))))); | 
| 38917 | 160 | |
| 24219 | 161 | |
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 162 | (* serializers: functions producing serializations *) | 
| 28054 | 163 | |
| 39142 | 164 | type serializer = Token.T list | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 165 | -> Proof.context | 
| 39142 | 166 |   -> {
 | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 167 | module_name: string, | 
| 38926 | 168 | reserved_syms: string list, | 
| 59103 | 169 | identifiers: Code_Printer.identifiers, | 
| 38926 | 170 | includes: (string * Pretty.T) list, | 
| 171 | class_syntax: string -> string option, | |
| 172 | tyco_syntax: string -> Code_Printer.tyco_syntax option, | |
| 55153 
eedd549de3ef
more suitable names, without any notion of "activating"
 haftmann parents: 
55150diff
changeset | 173 | const_syntax: string -> Code_Printer.const_syntax option } | 
| 55683 | 174 | -> Code_Symbol.T list | 
| 41342 
3519e0dd8f75
more explicit structure for serializer invocation
 haftmann parents: 
41307diff
changeset | 175 | -> Code_Thingol.program | 
| 28054 | 176 | -> serialization; | 
| 27000 | 177 | |
| 59102 | 178 | |
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 179 | (** theory data **) | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 180 | |
| 59102 | 181 | type language = { serializer: serializer, literals: literals,
 | 
| 182 |   check: { env_var: string, make_destination: Path.T -> Path.T, make_command: string -> string } }; 
 | |
| 183 | ||
| 59103 | 184 | type ancestry = (string * (Code_Thingol.program -> Code_Thingol.program)) list; | 
| 27103 | 185 | |
| 59103 | 186 | val merge_ancestry : ancestry * ancestry -> ancestry = AList.join (op =) (K snd); | 
| 27103 | 187 | |
| 59103 | 188 | type target = { serial: serial, language: language, ancestry: ancestry };
 | 
| 27437 | 189 | |
| 34248 | 190 | structure Targets = Theory_Data | 
| 34071 | 191 | ( | 
| 59324 | 192 | type T = (target * Code_Printer.data) Symtab.table; | 
| 193 | val empty = Symtab.empty; | |
| 34071 | 194 | val extend = I; | 
| 59324 | 195 | fun merge (targets1, targets2) : T = | 
| 196 | Symtab.join (fn target_name => fn ((target1, data1), (target2, data2)) => | |
| 59103 | 197 | if #serial target1 = #serial target2 then | 
| 198 |       ({ serial = #serial target1, language = #language target1,
 | |
| 199 | ancestry = merge_ancestry (#ancestry target1, #ancestry target2)}, | |
| 200 | Code_Printer.merge_data (data1, data2)) | |
| 59102 | 201 |       else error ("Incompatible targets: " ^ quote target_name) 
 | 
| 59324 | 202 | ) (targets1, targets2) | 
| 34071 | 203 | ); | 
| 27436 | 204 | |
| 59324 | 205 | fun exists_target thy = Symtab.defined (Targets.get thy); | 
| 206 | fun lookup_target_data thy = Symtab.lookup (Targets.get thy); | |
| 59479 | 207 | fun assert_target thy target_name = | 
| 208 | if exists_target thy target_name | |
| 209 | then target_name | |
| 210 |   else error ("Unknown code target language: " ^ quote target_name);
 | |
| 59100 | 211 | |
| 59104 | 212 | fun fold1 f xs = fold f (tl xs) (hd xs); | 
| 213 | ||
| 59101 
6dc48c98303c
tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
 haftmann parents: 
59100diff
changeset | 214 | fun join_ancestry thy target_name = | 
| 
6dc48c98303c
tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
 haftmann parents: 
59100diff
changeset | 215 | let | 
| 59479 | 216 | val _ = assert_target thy target_name; | 
| 59103 | 217 | val the_target_data = the o lookup_target_data thy; | 
| 218 | val (target, this_data) = the_target_data target_name; | |
| 219 | val ancestry = #ancestry target; | |
| 59102 | 220 | val modifies = rev (map snd ancestry); | 
| 221 | val modify = fold (curry (op o)) modifies I; | |
| 59103 | 222 | val datas = rev (map (snd o the_target_data o fst) ancestry) @ [this_data]; | 
| 59104 | 223 | val data = fold1 (fn data' => fn data => Code_Printer.merge_data (data, data')) datas; | 
| 59103 | 224 | in (modify, (target, data)) end; | 
| 59101 
6dc48c98303c
tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
 haftmann parents: 
59100diff
changeset | 225 | |
| 59479 | 226 | fun allocate_target target_name target thy = | 
| 27304 | 227 | let | 
| 59101 
6dc48c98303c
tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
 haftmann parents: 
59100diff
changeset | 228 | val _ = if exists_target thy target_name | 
| 
6dc48c98303c
tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
 haftmann parents: 
59100diff
changeset | 229 |       then error ("Attempt to overwrite existing target " ^ quote target_name)
 | 
| 43564 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43324diff
changeset | 230 | else (); | 
| 28054 | 231 | in | 
| 232 | thy | |
| 59324 | 233 | |> (Targets.map o Symtab.update) (target_name, (target, Code_Printer.empty_data)) | 
| 28054 | 234 | end; | 
| 27436 | 235 | |
| 59104 | 236 | fun add_language (target_name, language) = | 
| 59102 | 237 |   allocate_target target_name { serial = serial (), language = language, ancestry = [] };
 | 
| 27436 | 238 | |
| 59104 | 239 | fun add_derived_target (target_name, initial_ancestry) thy = | 
| 59101 
6dc48c98303c
tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
 haftmann parents: 
59100diff
changeset | 240 | let | 
| 59104 | 241 | val _ = if null initial_ancestry | 
| 242 | then error "Must derive from existing target(s)" else (); | |
| 243 | fun the_target_data target_name' = case lookup_target_data thy target_name' of | |
| 244 |       NONE => error ("Unknown code target language: " ^ quote target_name')
 | |
| 245 | | SOME target_data' => target_data'; | |
| 246 | val targets = rev (map (fst o the_target_data o fst) initial_ancestry); | |
| 247 | val supremum = fold1 (fn target' => fn target => | |
| 248 | if #serial target = #serial target' | |
| 249 | then target else error "Incompatible targets") targets; | |
| 250 | val ancestries = map #ancestry targets @ [initial_ancestry]; | |
| 251 | val ancestry = fold1 (fn ancestry' => fn ancestry => | |
| 252 | merge_ancestry (ancestry, ancestry')) ancestries; | |
| 59101 
6dc48c98303c
tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
 haftmann parents: 
59100diff
changeset | 253 | in | 
| 59104 | 254 |     allocate_target target_name { serial = #serial supremum, language = #language supremum,
 | 
| 255 | ancestry = ancestry } thy | |
| 59101 
6dc48c98303c
tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
 haftmann parents: 
59100diff
changeset | 256 | end; | 
| 
6dc48c98303c
tuned target inheritance bookkeeping: ancestry is always fully maintained at current entry using canonical merge;
 haftmann parents: 
59100diff
changeset | 257 | |
| 59102 | 258 | fun map_data target_name f thy = | 
| 27436 | 259 | let | 
| 59479 | 260 | val _ = assert_target thy target_name; | 
| 28054 | 261 | in | 
| 262 | thy | |
| 59324 | 263 | |> (Targets.map o Symtab.map_entry target_name o apsnd o Code_Printer.map_data) f | 
| 28054 | 264 | end; | 
| 27304 | 265 | |
| 59099 | 266 | fun map_reserved target_name = | 
| 59102 | 267 |   map_data target_name o @{apply 3 (1)};
 | 
| 59099 | 268 | fun map_identifiers target_name = | 
| 59102 | 269 |   map_data target_name o @{apply 3 (2)};
 | 
| 59099 | 270 | fun map_printings target_name = | 
| 59102 | 271 |   map_data target_name o @{apply 3 (3)};
 | 
| 27000 | 272 | |
| 273 | ||
| 34021 | 274 | (** serializer usage **) | 
| 275 | ||
| 59324 | 276 | (* technical aside: pretty printing width *) | 
| 277 | ||
| 278 | val default_code_width = Attrib.setup_config_int @{binding "default_code_width"} (K 80);
 | |
| 279 | ||
| 280 | ||
| 34021 | 281 | (* montage *) | 
| 282 | ||
| 59102 | 283 | fun the_language ctxt = | 
| 59103 | 284 | #language o fst o the o lookup_target_data (Proof_Context.theory_of ctxt); | 
| 37822 
cf3588177676
use generic description slot for formal code checking
 haftmann parents: 
37821diff
changeset | 285 | |
| 59102 | 286 | fun the_literals ctxt = #literals o the_language ctxt; | 
| 34021 | 287 | |
| 39817 
5228c6b20273
check whole target hierarchy for existing reserved symbols
 haftmann parents: 
39750diff
changeset | 288 | local | 
| 
5228c6b20273
check whole target hierarchy for existing reserved symbols
 haftmann parents: 
39750diff
changeset | 289 | |
| 59099 | 290 | fun activate_target ctxt target_name = | 
| 39817 
5228c6b20273
check whole target hierarchy for existing reserved symbols
 haftmann parents: 
39750diff
changeset | 291 | let | 
| 59324 | 292 | val thy = Proof_Context.theory_of ctxt; | 
| 59103 | 293 | val (modify, target_data) = join_ancestry thy target_name; | 
| 59324 | 294 | in (target_data, modify) end; | 
| 38927 | 295 | |
| 55757 | 296 | fun project_program ctxt syms_hidden syms1 program2 = | 
| 38927 | 297 | let | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 298 | val syms2 = subtract (op =) syms_hidden syms1; | 
| 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 299 | val program3 = Code_Symbol.Graph.restrict (not o member (op =) syms_hidden) program2; | 
| 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 300 | val syms4 = Code_Symbol.Graph.all_succs program3 syms2; | 
| 54890 
cb892d835803
fundamental treatment of undefined vs. universally partial replaces code_abort
 haftmann parents: 
54889diff
changeset | 301 | val unimplemented = Code_Thingol.unimplemented program3; | 
| 42359 | 302 | val _ = | 
| 54889 
4121d64fde90
explicit distinction between empty code equations and no code equations, including convenient declaration attributes
 haftmann parents: 
54312diff
changeset | 303 | if null unimplemented then () | 
| 42359 | 304 |       else error ("No code equations for " ^
 | 
| 55304 | 305 | commas (map (Proof_Context.markup_const ctxt) unimplemented)); | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 306 | val program4 = Code_Symbol.Graph.restrict (member (op =) syms4) program3; | 
| 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 307 | in (syms4, program4) end; | 
| 38927 | 308 | |
| 55757 | 309 | fun prepare_serializer ctxt (serializer : serializer) reserved identifiers | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 310 | printings module_name args proto_program syms = | 
| 38927 | 311 | let | 
| 55149 
626d8f08d479
immediate "activation" of const syntax at declaration time
 haftmann parents: 
55147diff
changeset | 312 | val syms_hidden = Code_Symbol.symbols_of printings; | 
| 55757 | 313 | val (syms_all, program) = project_program ctxt syms_hidden syms proto_program; | 
| 39484 
505f95975a5a
closures separate serializer initialization from serializer invocation as far as appropriate
 haftmann parents: 
39480diff
changeset | 314 | fun select_include (name, (content, cs)) = | 
| 55150 | 315 | if null cs orelse exists (fn c => member (op =) syms_all (Constant c)) cs | 
| 39484 
505f95975a5a
closures separate serializer initialization from serializer invocation as far as appropriate
 haftmann parents: 
39480diff
changeset | 316 | then SOME (name, content) else NONE; | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 317 | val includes = map_filter select_include (Code_Symbol.dest_module_data printings); | 
| 34021 | 318 | in | 
| 55757 | 319 |     (serializer args ctxt {
 | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 320 | module_name = module_name, | 
| 38926 | 321 | reserved_syms = reserved, | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 322 | identifiers = identifiers, | 
| 38926 | 323 | includes = includes, | 
| 55149 
626d8f08d479
immediate "activation" of const syntax at declaration time
 haftmann parents: 
55147diff
changeset | 324 | const_syntax = Code_Symbol.lookup_constant_data printings, | 
| 
626d8f08d479
immediate "activation" of const syntax at declaration time
 haftmann parents: 
55147diff
changeset | 325 | tyco_syntax = Code_Symbol.lookup_type_constructor_data printings, | 
| 
626d8f08d479
immediate "activation" of const syntax at declaration time
 haftmann parents: 
55147diff
changeset | 326 | class_syntax = Code_Symbol.lookup_type_class_data printings }, | 
| 55776 
7dd1971b39c1
amended some slips, rolling back currently dysfunctional export minimimalisation for Scala
 haftmann parents: 
55757diff
changeset | 327 | (subtract (op =) syms_hidden syms, program)) | 
| 34021 | 328 | end; | 
| 329 | ||
| 59099 | 330 | fun mount_serializer ctxt target_name some_width module_name args program syms = | 
| 34021 | 331 | let | 
| 59324 | 332 | val default_width = Config.get ctxt default_code_width; | 
| 333 | val ((target, data), modify) = activate_target ctxt target_name; | |
| 59103 | 334 | val serializer = (#serializer o #language) target; | 
| 55683 | 335 | val (prepared_serializer, (prepared_syms, prepared_program)) = | 
| 55757 | 336 | prepare_serializer ctxt serializer | 
| 59103 | 337 | (Code_Printer.the_reserved data) (Code_Printer.the_identifiers data) | 
| 338 | (Code_Printer.the_printings data) | |
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 339 | module_name args (modify program) syms | 
| 34071 | 340 | val width = the_default default_width some_width; | 
| 55683 | 341 | in (fn program => fn syms => prepared_serializer syms program width, (prepared_syms, prepared_program)) end; | 
| 41344 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 342 | |
| 59099 | 343 | fun invoke_serializer ctxt target_name some_width raw_module_name args program all_public syms = | 
| 41344 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 344 | let | 
| 55291 | 345 | val module_name = if raw_module_name = "" then "" | 
| 346 | else (check_name true raw_module_name; raw_module_name) | |
| 55757 | 347 | val (mounted_serializer, (prepared_syms, prepared_program)) = | 
| 59099 | 348 | mount_serializer ctxt target_name some_width module_name args program syms; | 
| 63164 | 349 | in | 
| 350 | Code_Preproc.timed_exec "serializing" | |
| 351 | (fn () => mounted_serializer prepared_program (if all_public then [] else prepared_syms)) ctxt | |
| 352 | end; | |
| 34021 | 353 | |
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 354 | fun assert_module_name "" = error "Empty module name not allowed here" | 
| 38933 
bd77e092f67c
avoid strange special treatment of empty module names
 haftmann parents: 
38929diff
changeset | 355 | | assert_module_name module_name = module_name; | 
| 
bd77e092f67c
avoid strange special treatment of empty module names
 haftmann parents: 
38929diff
changeset | 356 | |
| 62550 | 357 | val using_master_directory = | 
| 358 | Option.map o File.full_path o Resources.master_directory o Proof_Context.theory_of; | |
| 48371 | 359 | |
| 34021 | 360 | in | 
| 361 | ||
| 48568 | 362 | val generatedN = "Generated_Code"; | 
| 363 | ||
| 59099 | 364 | fun export_code_for ctxt some_path target_name some_width module_name args = | 
| 55757 | 365 | export (using_master_directory ctxt some_path) | 
| 59099 | 366 | ooo invoke_serializer ctxt target_name some_width module_name args; | 
| 38918 | 367 | |
| 59099 | 368 | fun produce_code_for ctxt target_name some_width module_name args = | 
| 39102 | 369 | let | 
| 59099 | 370 | val serializer = invoke_serializer ctxt target_name some_width (assert_module_name module_name) args; | 
| 55683 | 371 | in fn program => fn all_public => fn syms => | 
| 372 | produce (serializer program all_public syms) |> apsnd (fn deresolve => map deresolve syms) | |
| 39484 
505f95975a5a
closures separate serializer initialization from serializer invocation as far as appropriate
 haftmann parents: 
39480diff
changeset | 373 | end; | 
| 38929 
d9ac9dee764d
distinguish code production and code presentation
 haftmann parents: 
38928diff
changeset | 374 | |
| 59099 | 375 | fun present_code_for ctxt target_name some_width module_name args = | 
| 39484 
505f95975a5a
closures separate serializer initialization from serializer invocation as far as appropriate
 haftmann parents: 
39480diff
changeset | 376 | let | 
| 59099 | 377 | val serializer = invoke_serializer ctxt target_name some_width (assert_module_name module_name) args; | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 378 | in fn program => fn (syms, selects) => | 
| 55683 | 379 | present selects (serializer program false syms) | 
| 39484 
505f95975a5a
closures separate serializer initialization from serializer invocation as far as appropriate
 haftmann parents: 
39480diff
changeset | 380 | end; | 
| 38918 | 381 | |
| 59099 | 382 | fun check_code_for ctxt target_name strict args program all_public syms = | 
| 37824 | 383 | let | 
| 384 |     val { env_var, make_destination, make_command } =
 | |
| 59102 | 385 | (#check o the_language ctxt) target_name; | 
| 41939 | 386 | fun ext_check p = | 
| 43564 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43324diff
changeset | 387 | let | 
| 37824 | 388 | val destination = make_destination p; | 
| 59099 | 389 | val _ = export (SOME destination) (invoke_serializer ctxt target_name (SOME 80) | 
| 55683 | 390 | generatedN args program all_public syms); | 
| 48568 | 391 | val cmd = make_command generatedN; | 
| 43850 
7f2cbc713344
moved bash operations to Isabelle_System (cf. Scala version);
 wenzelm parents: 
43564diff
changeset | 392 | in | 
| 62549 
9498623b27f0
File.bash_string operations in ML as in Scala -- exclusively for GNU bash, not perl and not user output;
 wenzelm parents: 
59936diff
changeset | 393 |         if Isabelle_System.bash ("cd " ^ File.bash_path p ^ " && " ^ cmd ^ " 2>&1") <> 0
 | 
| 59099 | 394 |         then error ("Code check failed for " ^ target_name ^ ": " ^ cmd)
 | 
| 37824 | 395 | else () | 
| 396 | end; | |
| 43850 
7f2cbc713344
moved bash operations to Isabelle_System (cf. Scala version);
 wenzelm parents: 
43564diff
changeset | 397 | in | 
| 63024 
adeac19dd410
environment variable check has become pointless after 771b8ad5c7fc
 haftmann parents: 
62969diff
changeset | 398 | if not (env_var = "") andalso getenv env_var = "" | 
| 37825 | 399 | then if strict | 
| 59099 | 400 | then error (env_var ^ " not set; cannot check code for " ^ target_name) | 
| 401 | else warning (env_var ^ " not set; skipped checking code for " ^ target_name) | |
| 41939 | 402 | else Isabelle_System.with_tmp_dir "Code_Test" ext_check | 
| 37824 | 403 | end; | 
| 404 | ||
| 64957 | 405 | fun dynamic_compilation_text mounted_serializer prepared_program syms all_public ((vs, ty), t) = | 
| 41344 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 406 | let | 
| 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 407 | val _ = if Code_Thingol.contains_dict_var t then | 
| 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 408 | error "Term to be evaluated contains free dictionaries" else (); | 
| 43324 
2b47822868e4
discontinued Name.variant to emphasize that this is old-style / indirect;
 wenzelm parents: 
42361diff
changeset | 409 | val v' = singleton (Name.variant_list (map fst vs)) "a"; | 
| 41344 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 410 | val vs' = (v', []) :: vs; | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 411 | val ty' = ITyVar v' `-> ty; | 
| 41344 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 412 | val program = prepared_program | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 413 | |> Code_Symbol.Graph.new_node (Code_Symbol.value, | 
| 57249 
5c75baf68b77
formal variable name: IVar NONE is strictly spoken not supported on lhs of function definitions, e.g. in Scala
 haftmann parents: 
56920diff
changeset | 414 | Code_Thingol.Fun (((vs', ty'), [(([IVar (SOME "dummy")], t), (NONE, true))]), NONE)) | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 415 | |> fold (curry (perhaps o try o | 
| 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 416 | Code_Symbol.Graph.add_edge) Code_Symbol.value) syms; | 
| 55683 | 417 | val (program_code, deresolve) = | 
| 55684 
ee49b4f7edc8
keep only identifiers public which are explicitly requested or demanded by dependencies
 haftmann parents: 
55683diff
changeset | 418 | produce (mounted_serializer program (if all_public then [] else [Code_Symbol.value])); | 
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 419 | val value_name = the (deresolve Code_Symbol.value); | 
| 64959 | 420 | in ((program_code, value_name), deresolve) end; | 
| 41344 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 421 | |
| 64959 | 422 | fun compilation_text' ctxt target_name some_module_name program syms = | 
| 41344 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 423 | let | 
| 55683 | 424 | val (mounted_serializer, (_, prepared_program)) = | 
| 64959 | 425 | mount_serializer ctxt target_name NONE (the_default generatedN some_module_name) [] program syms; | 
| 63164 | 426 | in | 
| 427 | Code_Preproc.timed_exec "serializing" | |
| 64957 | 428 | (fn () => dynamic_compilation_text mounted_serializer prepared_program syms) ctxt | 
| 63164 | 429 | end; | 
| 41344 
d990badc97a3
evaluator separating static and dynamic operations
 haftmann parents: 
41342diff
changeset | 430 | |
| 64959 | 431 | fun compilation_text ctxt target_name program syms = | 
| 432 | fst oo compilation_text' ctxt target_name NONE program syms | |
| 433 | ||
| 34021 | 434 | end; (* local *) | 
| 435 | ||
| 436 | ||
| 437 | (* code generation *) | |
| 438 | ||
| 38918 | 439 | fun prep_destination "" = NONE | 
| 440 | | prep_destination s = SOME (Path.explode s); | |
| 441 | ||
| 55757 | 442 | fun export_code ctxt all_public cs seris = | 
| 34021 | 443 | let | 
| 63159 | 444 | val program = Code_Thingol.consts_program ctxt cs; | 
| 59099 | 445 | val _ = map (fn (((target_name, module_name), some_path), args) => | 
| 446 | export_code_for ctxt some_path target_name NONE module_name args program all_public (map Constant cs)) seris; | |
| 34021 | 447 | in () end; | 
| 448 | ||
| 55757 | 449 | fun export_code_cmd all_public raw_cs seris ctxt = | 
| 450 | export_code ctxt all_public | |
| 451 | (Code_Thingol.read_const_exprs ctxt raw_cs) | |
| 55683 | 452 | ((map o apfst o apsnd) prep_destination seris); | 
| 38918 | 453 | |
| 59099 | 454 | fun produce_code ctxt all_public cs target_name some_width some_module_name args = | 
| 38918 | 455 | let | 
| 63159 | 456 | val program = Code_Thingol.consts_program ctxt cs; | 
| 59099 | 457 | in produce_code_for ctxt target_name some_width some_module_name args program all_public (map Constant cs) end; | 
| 38929 
d9ac9dee764d
distinguish code production and code presentation
 haftmann parents: 
38928diff
changeset | 458 | |
| 59099 | 459 | fun present_code ctxt cs syms target_name some_width some_module_name args = | 
| 38929 
d9ac9dee764d
distinguish code production and code presentation
 haftmann parents: 
38928diff
changeset | 460 | let | 
| 63159 | 461 | val program = Code_Thingol.consts_program ctxt cs; | 
| 59099 | 462 | in present_code_for ctxt target_name some_width some_module_name args program (map Constant cs, syms) end; | 
| 34021 | 463 | |
| 55757 | 464 | fun check_code ctxt all_public cs seris = | 
| 37824 | 465 | let | 
| 63159 | 466 | val program = Code_Thingol.consts_program ctxt cs; | 
| 59099 | 467 | val _ = map (fn ((target_name, strict), args) => | 
| 468 | check_code_for ctxt target_name strict args program all_public (map Constant cs)) seris; | |
| 37824 | 469 | in () end; | 
| 470 | ||
| 55757 | 471 | fun check_code_cmd all_public raw_cs seris ctxt = | 
| 472 | check_code ctxt all_public | |
| 473 | (Code_Thingol.read_const_exprs ctxt raw_cs) seris; | |
| 37824 | 474 | |
| 39480 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 475 | local | 
| 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 476 | |
| 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 477 | val parse_const_terms = Scan.repeat1 Args.term | 
| 55757 | 478 | >> (fn ts => fn ctxt => map (Code.check_const (Proof_Context.theory_of ctxt)) ts); | 
| 39480 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 479 | |
| 55147 
bce3dbc11f95
prefer explicit code symbol type over ad-hoc name mangling
 haftmann parents: 
55146diff
changeset | 480 | fun parse_names category parse internalize mark_symbol = | 
| 39480 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 481 | Scan.lift (Args.parens (Args.$$$ category)) |-- Scan.repeat1 parse | 
| 55757 | 482 | >> (fn xs => fn ctxt => map (mark_symbol o internalize ctxt) xs); | 
| 43564 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43324diff
changeset | 483 | |
| 39480 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 484 | val parse_consts = parse_names "consts" Args.term | 
| 55757 | 485 | (Code.check_const o Proof_Context.theory_of) Constant; | 
| 39480 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 486 | |
| 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 487 | val parse_types = parse_names "types" (Scan.lift Args.name) | 
| 55757 | 488 | (Sign.intern_type o Proof_Context.theory_of) Type_Constructor; | 
| 39480 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 489 | |
| 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 490 | val parse_classes = parse_names "classes" (Scan.lift Args.name) | 
| 55757 | 491 | (Sign.intern_class o Proof_Context.theory_of) Type_Class; | 
| 39480 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 492 | |
| 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 493 | val parse_instances = parse_names "instances" (Scan.lift (Args.name --| Args.$$$ "::" -- Args.name)) | 
| 55757 | 494 | (fn ctxt => fn (raw_tyco, raw_class) => | 
| 495 | let | |
| 496 | val thy = Proof_Context.theory_of ctxt; | |
| 497 | in (Sign.intern_class thy raw_tyco, Sign.intern_type thy raw_class) end) Class_Instance; | |
| 39480 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 498 | |
| 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 499 | in | 
| 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 500 | |
| 59323 | 501 | val _ = Theory.setup | 
| 502 |   (Thy_Output.antiquotation @{binding code_stmts}
 | |
| 43564 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43324diff
changeset | 503 | (parse_const_terms -- | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43324diff
changeset | 504 | Scan.repeat (parse_consts || parse_types || parse_classes || parse_instances) | 
| 
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
 wenzelm parents: 
43324diff
changeset | 505 | -- Scan.lift (Args.parens (Args.name -- Scan.option Parse.int))) | 
| 59099 | 506 |     (fn {context = ctxt, ...} => fn ((mk_cs, mk_stmtss), (target_name, some_width)) =>
 | 
| 55757 | 507 | present_code ctxt (mk_cs ctxt) | 
| 508 | (maps (fn f => f ctxt) mk_stmtss) | |
| 59323 | 509 | target_name some_width "Example" [])); | 
| 39480 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 510 | |
| 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 511 | end; | 
| 
a2ed61449dcc
added code_stmts antiquotation from doc-src/more_antiquote.ML
 haftmann parents: 
39142diff
changeset | 512 | |
| 34021 | 513 | |
| 28054 | 514 | (** serializer configuration **) | 
| 27000 | 515 | |
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 516 | (* reserved symbol names *) | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 517 | |
| 59099 | 518 | fun add_reserved target_name sym thy = | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 519 | let | 
| 59103 | 520 | val (_, (_, data)) = join_ancestry thy target_name; | 
| 521 | val _ = if member (op =) (Code_Printer.the_reserved data) sym | |
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 522 |       then error ("Reserved symbol " ^ quote sym ^ " already declared")
 | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 523 | else (); | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 524 | in | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 525 | thy | 
| 59099 | 526 | |> map_reserved target_name (insert (op =) sym) | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 527 | end; | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 528 | |
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 529 | |
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 530 | (* checking of syntax *) | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 531 | |
| 59099 | 532 | fun check_const_syntax ctxt target_name c syn = | 
| 55757 | 533 | if Code_Printer.requires_args syn > Code.args_number (Proof_Context.theory_of ctxt) c | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 534 |   then error ("Too many arguments in syntax for constant " ^ quote c)
 | 
| 59099 | 535 | else Code_Printer.prep_const_syntax (Proof_Context.theory_of ctxt) (the_literals ctxt target_name) c syn; | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 536 | |
| 59099 | 537 | fun check_tyco_syntax ctxt target_name tyco syn = | 
| 55757 | 538 | if fst syn <> Sign.arity_number (Proof_Context.theory_of ctxt) tyco | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 539 |   then error ("Number of arguments mismatch in syntax for type constructor " ^ quote tyco)
 | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 540 | else syn; | 
| 34071 | 541 | |
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 542 | |
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 543 | (* custom symbol names *) | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 544 | |
| 52218 | 545 | fun arrange_name_decls x = | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 546 | let | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 547 | fun arrange is_module (sym, target_names) = map (fn (target, some_name) => | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 548 | (target, (sym, Option.map (check_name is_module) some_name))) target_names; | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 549 | in | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 550 | Code_Symbol.maps_attr' (arrange false) (arrange false) (arrange false) | 
| 52218 | 551 | (arrange false) (arrange false) (arrange true) x | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 552 | end; | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 553 | |
| 55757 | 554 | fun cert_name_decls ctxt = cert_syms ctxt #> arrange_name_decls; | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 555 | |
| 55757 | 556 | fun read_name_decls ctxt = read_syms ctxt #> arrange_name_decls; | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 557 | |
| 59099 | 558 | fun set_identifier (target_name, sym_name) = map_identifiers target_name (Code_Symbol.set_data sym_name); | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 559 | |
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 560 | fun gen_set_identifiers prep_name_decl raw_name_decls thy = | 
| 55757 | 561 | fold set_identifier (prep_name_decl (Proof_Context.init_global thy) raw_name_decls) thy; | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 562 | |
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 563 | val set_identifiers = gen_set_identifiers cert_name_decls; | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 564 | val set_identifiers_cmd = gen_set_identifiers read_name_decls; | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 565 | |
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 566 | |
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 567 | (* custom printings *) | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 568 | |
| 55757 | 569 | fun arrange_printings prep_const ctxt = | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 570 | let | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 571 | fun arrange check (sym, target_syns) = | 
| 59099 | 572 | map (fn (target_name, some_syn) => | 
| 573 | (target_name, (sym, Option.map (check ctxt target_name sym) some_syn))) target_syns; | |
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 574 | in | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 575 | Code_Symbol.maps_attr' | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 576 | (arrange check_const_syntax) (arrange check_tyco_syntax) | 
| 55149 
626d8f08d479
immediate "activation" of const syntax at declaration time
 haftmann parents: 
55147diff
changeset | 577 | (arrange ((K o K o K) I)) (arrange ((K o K o K) I)) (arrange ((K o K o K) I)) | 
| 55757 | 578 | (arrange (fn ctxt => fn _ => fn _ => fn (raw_content, raw_cs) => | 
| 59430 | 579 | (Pretty.blk (0, Pretty.fbreaks (map Code_Printer.str (split_lines raw_content))), | 
| 580 | map (prep_const ctxt) raw_cs))) | |
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 581 | end; | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 582 | |
| 55757 | 583 | fun cert_printings ctxt = cert_syms ctxt #> arrange_printings cert_const ctxt; | 
| 24219 | 584 | |
| 55757 | 585 | fun read_printings ctxt = read_syms ctxt #> arrange_printings read_const ctxt; | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 586 | |
| 59099 | 587 | fun set_printing (target_name, sym_syn) = map_printings target_name (Code_Symbol.set_data sym_syn); | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 588 | |
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 589 | fun gen_set_printings prep_print_decl raw_print_decls thy = | 
| 55757 | 590 | fold set_printing (prep_print_decl (Proof_Context.init_global thy) raw_print_decls) thy; | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 591 | |
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 592 | val set_printings = gen_set_printings cert_printings; | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 593 | val set_printings_cmd = gen_set_printings read_printings; | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 594 | |
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 595 | |
| 27103 | 596 | (* concrete syntax *) | 
| 27000 | 597 | |
| 28054 | 598 | fun parse_args f args = | 
| 36959 
f5417836dbea
renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
 wenzelm parents: 
36537diff
changeset | 599 | case Scan.read Token.stopper f args | 
| 28054 | 600 | of SOME x => x | 
| 601 | | NONE => error "Bad serializer arguments"; | |
| 602 | ||
| 603 | ||
| 27304 | 604 | (** Isar setup **) | 
| 27103 | 605 | |
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 606 | fun parse_single_symbol_pragma parse_keyword parse_isa parse_target = | 
| 52434 | 607 |   parse_keyword |-- Parse.!!! (parse_isa --| (@{keyword "\<rightharpoonup>"} || @{keyword "=>"})
 | 
| 608 |     -- Parse.and_list1 (@{keyword "("} |-- (Parse.name --| @{keyword ")"} -- Scan.option parse_target)));
 | |
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 609 | |
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 610 | fun parse_symbol_pragma parse_const parse_tyco parse_class parse_classrel parse_inst parse_module = | 
| 52801 | 611 |   parse_single_symbol_pragma @{keyword "constant"} Parse.term parse_const
 | 
| 55150 | 612 | >> Constant | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 613 |   || parse_single_symbol_pragma @{keyword "type_constructor"} Parse.type_const parse_tyco
 | 
| 55150 | 614 | >> Type_Constructor | 
| 52377 
afa72aaed518
more consistent parsing and reading of classes and type constructors
 haftmann parents: 
52218diff
changeset | 615 |   || parse_single_symbol_pragma @{keyword "type_class"} Parse.class parse_class
 | 
| 55150 | 616 | >> Type_Class | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 617 |   || parse_single_symbol_pragma @{keyword "class_relation"} parse_classrel_ident parse_classrel
 | 
| 55150 | 618 | >> Class_Relation | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 619 |   || parse_single_symbol_pragma @{keyword "class_instance"} parse_inst_ident parse_inst
 | 
| 55150 | 620 | >> Class_Instance | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 621 |   || parse_single_symbol_pragma @{keyword "code_module"} Parse.name parse_module
 | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 622 | >> Code_Symbol.Module; | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 623 | |
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 624 | fun parse_symbol_pragmas parse_const parse_tyco parse_class parse_classrel parse_inst parse_module = | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 625 | Parse.enum1 "|" (Parse.group (fn () => "code symbol pragma") | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 626 | (parse_symbol_pragma parse_const parse_tyco parse_class parse_classrel parse_inst parse_module)); | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 627 | |
| 56201 | 628 | val code_expr_argsP = Scan.optional (@{keyword "("} |-- Parse.args --| @{keyword ")"}) [];
 | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 629 | |
| 55683 | 630 | fun code_expr_inP all_public raw_cs = | 
| 52434 | 631 |   Scan.repeat (@{keyword "in"} |-- Parse.!!! (Parse.name
 | 
| 632 |     -- Scan.optional (@{keyword "module_name"} |-- Parse.name) ""
 | |
| 633 |     -- Scan.optional (@{keyword "file"} |-- Parse.name) ""
 | |
| 634 | -- code_expr_argsP)) | |
| 55683 | 635 | >> (fn seri_args => export_code_cmd all_public raw_cs seri_args); | 
| 52434 | 636 | |
| 55683 | 637 | fun code_expr_checkingP all_public raw_cs = | 
| 52434 | 638 |   (@{keyword "checking"} |-- Parse.!!!
 | 
| 639 |     (Scan.repeat (Parse.name -- ((@{keyword "?"} |-- Scan.succeed false) || Scan.succeed true)
 | |
| 640 | -- code_expr_argsP))) | |
| 55683 | 641 | >> (fn seri_args => check_code_cmd all_public raw_cs seri_args); | 
| 52434 | 642 | |
| 55683 | 643 | val code_exprP = (Scan.optional (@{keyword "open"} |-- Scan.succeed true) false
 | 
| 644 | -- Scan.repeat1 Parse.term) | |
| 645 | :|-- (fn (all_public, raw_cs) => (code_expr_checkingP all_public raw_cs || code_expr_inP all_public raw_cs)); | |
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 646 | |
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 647 | val _ = | 
| 59936 
b8ffc3dc9e24
@{command_spec} is superseded by @{command_keyword};
 wenzelm parents: 
59480diff
changeset | 648 |   Outer_Syntax.command @{command_keyword code_reserved}
 | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 649 | "declare words as reserved for target language" | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 650 | (Parse.name -- Scan.repeat1 Parse.name | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 651 | >> (fn (target, reserveds) => (Toplevel.theory o fold (add_reserved target)) reserveds)); | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 652 | |
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 653 | val _ = | 
| 59936 
b8ffc3dc9e24
@{command_spec} is superseded by @{command_keyword};
 wenzelm parents: 
59480diff
changeset | 654 |   Outer_Syntax.command @{command_keyword code_identifier} "declare mandatory names for code symbols"
 | 
| 52138 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 655 | (parse_symbol_pragmas Parse.name Parse.name Parse.name Parse.name Parse.name Parse.name | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 656 | >> (Toplevel.theory o fold set_identifiers_cmd)); | 
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 657 | |
| 
e21426f244aa
bookkeeping and input syntax for exact specification of names of symbols in generated code
 haftmann parents: 
52137diff
changeset | 658 | val _ = | 
| 59936 
b8ffc3dc9e24
@{command_spec} is superseded by @{command_keyword};
 wenzelm parents: 
59480diff
changeset | 659 |   Outer_Syntax.command @{command_keyword code_printing} "declare dedicated printing for code symbols"
 | 
| 52137 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 660 | (parse_symbol_pragmas (Code_Printer.parse_const_syntax) (Code_Printer.parse_tyco_syntax) | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 661 | Parse.string (Parse.minus >> K ()) (Parse.minus >> K ()) | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 662 |       (Parse.text -- Scan.optional (@{keyword "attach"} |-- Scan.repeat1 Parse.term) [])
 | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 663 | >> (Toplevel.theory o fold set_printings_cmd)); | 
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 664 | |
| 
7f7337447b1b
use generic data for code symbols for unified "code_printing" syntax for custom serialisations
 haftmann parents: 
52068diff
changeset | 665 | val _ = | 
| 59936 
b8ffc3dc9e24
@{command_spec} is superseded by @{command_keyword};
 wenzelm parents: 
59480diff
changeset | 666 |   Outer_Syntax.command @{command_keyword export_code} "generate executable code for constants"
 | 
| 55757 | 667 | (Parse.!!! code_exprP >> (fn f => Toplevel.keep (f o Toplevel.context_of))); | 
| 30494 
c150e6fa4e0d
consider exit status of code generation direcitve
 haftmann parents: 
30242diff
changeset | 668 | |
| 24219 | 669 | end; (*struct*) |