| author | nipkow | 
| Tue, 31 Mar 2020 15:51:15 +0200 | |
| changeset 71633 | 07bec530f02e | 
| parent 69593 | 3dda49e08b9d | 
| child 82380 | ceb4f33d3073 | 
| permissions | -rw-r--r-- | 
| 68028 | 1 | (* Title: HOL/Tools/literal.ML | 
| 2 | Author: Florian Haftmann, TU Muenchen | |
| 3 | ||
| 4 | Logical and syntactic operations on literals (see also HOL/Tools/hologic.ML). | |
| 5 | *) | |
| 6 | ||
| 7 | signature LITERAL = | |
| 8 | sig | |
| 9 | val add_code: string -> theory -> theory | |
| 10 | end | |
| 11 | ||
| 12 | structure Literal: LITERAL = | |
| 13 | struct | |
| 14 | ||
| 15 | datatype character = datatype String_Syntax.character; | |
| 16 | ||
| 69593 | 17 | fun mk_literal_syntax [] = Syntax.const \<^const_syntax>\<open>String.empty_literal\<close> | 
| 68028 | 18 | | mk_literal_syntax (c :: cs) = | 
| 69593 | 19 | list_comb (Syntax.const \<^const_syntax>\<open>String.Literal\<close>, String_Syntax.mk_bits_syntax 7 c) | 
| 68028 | 20 | $ mk_literal_syntax cs; | 
| 21 | ||
| 22 | val dest_literal_syntax = | |
| 23 | let | |
| 69593 | 24 | fun dest (Const (\<^const_syntax>\<open>String.empty_literal\<close>, _)) = [] | 
| 25 | | dest (Const (\<^const_syntax>\<open>String.Literal\<close>, _) $ b0 $ b1 $ b2 $ b3 $ b4 $ b5 $ b6 $ t) = | |
| 68028 | 26 | String_Syntax.classify_character (String_Syntax.dest_bits_syntax [b0, b1, b2, b3, b4, b5, b6]) :: dest t | 
| 27 | | dest t = raise Match; | |
| 28 | in dest end; | |
| 29 | ||
| 69593 | 30 | fun ascii_tr [(c as Const (\<^syntax_const>\<open>_constrain\<close>, _)) $ t $ u] = | 
| 68028 | 31 | c $ ascii_tr [t] $ u | 
| 32 | | ascii_tr [Const (num, _)] = | |
| 33 | (mk_literal_syntax o single o (fn n => n mod 128) o #value o Lexicon.read_num) num | |
| 34 |   | ascii_tr ts = raise TERM ("ascii_tr", ts);
 | |
| 35 | ||
| 69593 | 36 | fun literal_tr [(c as Const (\<^syntax_const>\<open>_constrain\<close>, _)) $ t $ u] = | 
| 68028 | 37 | c $ literal_tr [t] $ u | 
| 38 | | literal_tr [Free (str, _)] = | |
| 68940 
25b431feb2e9
more appropriate conversion of HOL character literals to character codes: symbolic newline is interpreted as 0x10
 haftmann parents: 
68028diff
changeset | 39 | (mk_literal_syntax o map String_Syntax.ascii_ord_of o String_Syntax.plain_strings_of) str | 
| 68028 | 40 |   | literal_tr ts = raise TERM ("literal_tr", ts);
 | 
| 41 | ||
| 69593 | 42 | fun ascii k = Syntax.const \<^syntax_const>\<open>_Ascii\<close> | 
| 68028 | 43 | $ Syntax.free (String_Syntax.hex k); | 
| 44 | ||
| 69593 | 45 | fun literal cs = Syntax.const \<^syntax_const>\<open>_Literal\<close> | 
| 68028 | 46 | $ Syntax.const (Lexicon.implode_str cs); | 
| 47 | ||
| 48 | fun empty_literal_tr' _ = literal []; | |
| 49 | ||
| 50 | fun literal_tr' [b0, b1, b2, b3, b4, b5, b6, t] = | |
| 51 | let | |
| 52 | val cs = | |
| 69593 | 53 | dest_literal_syntax (list_comb (Syntax.const \<^const_syntax>\<open>String.Literal\<close>, [b0, b1, b2, b3, b4, b5, b6, t])) | 
| 68028 | 54 | fun is_printable (Char _) = true | 
| 55 | | is_printable (Ord _) = false; | |
| 56 | fun the_char (Char c) = c; | |
| 57 | fun the_ascii [Ord i] = i; | |
| 58 | in | |
| 59 | if forall is_printable cs | |
| 60 | then literal (map the_char cs) | |
| 61 | else if length cs = 1 | |
| 62 | then ascii (the_ascii cs) | |
| 63 | else raise Match | |
| 64 | end | |
| 65 | | literal_tr' _ = raise Match; | |
| 66 | ||
| 67 | open Basic_Code_Thingol; | |
| 68 | ||
| 69 | fun map_partial g f = | |
| 70 | let | |
| 71 | fun mapp [] = SOME [] | |
| 72 | | mapp (x :: xs) = | |
| 73 | (case f x of | |
| 74 | NONE => NONE | |
| 75 | | SOME y => | |
| 76 | (case mapp xs of | |
| 77 | NONE => NONE | |
| 78 | | SOME ys => SOME (y :: ys))) | |
| 79 | in Option.map g o mapp end; | |
| 80 | ||
| 69593 | 81 | fun implode_bit (IConst { sym = Code_Symbol.Constant \<^const_name>\<open>False\<close>, ... }) = SOME 0
 | 
| 82 |   | implode_bit (IConst { sym = Code_Symbol.Constant \<^const_name>\<open>True\<close>, ... }) = SOME 1
 | |
| 68028 | 83 | | implode_bit _ = NONE | 
| 84 | ||
| 85 | fun implode_ascii (b0, b1, b2, b3, b4, b5, b6) = | |
| 86 | map_partial (chr o Integer.eval_radix 2) implode_bit [b0, b1, b2, b3, b4, b5, b6]; | |
| 87 | ||
| 88 | fun implode_literal b0 b1 b2 b3 b4 b5 b6 t = | |
| 89 | let | |
| 69593 | 90 |     fun dest_literal (IConst { sym = Code_Symbol.Constant \<^const_name>\<open>String.Literal\<close>, ... }
 | 
| 68028 | 91 | `$ b0 `$ b1 `$ b2 `$ b3 `$ b4 `$ b5 `$ b6 `$ t) = SOME ((b0, b1, b2, b3, b4, b5, b6), t) | 
| 92 | | dest_literal _ = NONE; | |
| 93 | val (bss', t') = Code_Thingol.unfoldr dest_literal t; | |
| 94 | val bss = (b0, b1, b2, b3, b4, b5, b6) :: bss'; | |
| 95 | in | |
| 96 | case t' of | |
| 69593 | 97 |       IConst { sym = Code_Symbol.Constant \<^const_name>\<open>String.zero_literal_inst.zero_literal\<close>, ... }
 | 
| 68028 | 98 | => map_partial implode implode_ascii bss | 
| 99 | | _ => NONE | |
| 100 | end; | |
| 101 | ||
| 102 | fun add_code target thy = | |
| 103 | let | |
| 104 | fun pretty literals _ thm _ _ [(b0, _), (b1, _), (b2, _), (b3, _), (b4, _), (b5, _), (b6, _), (t, _)] = | |
| 105 | case implode_literal b0 b1 b2 b3 b4 b5 b6 t of | |
| 106 | SOME s => (Code_Printer.str o Code_Printer.literal_string literals) s | |
| 107 | | NONE => Code_Printer.eqn_error thy thm "Illegal string literal expression"; | |
| 108 | in | |
| 109 | thy | |
| 69593 | 110 | |> Code_Target.set_printings (Code_Symbol.Constant (\<^const_name>\<open>String.Literal\<close>, | 
| 68028 | 111 | [(target, SOME (Code_Printer.complex_const_syntax (8, pretty)))])) | 
| 112 | end; | |
| 113 | ||
| 114 | val _ = | |
| 115 | Theory.setup | |
| 116 | (Sign.parse_translation | |
| 69593 | 117 | [(\<^syntax_const>\<open>_Ascii\<close>, K ascii_tr), | 
| 118 | (\<^syntax_const>\<open>_Literal\<close>, K literal_tr)] #> | |
| 68028 | 119 | Sign.print_translation | 
| 69593 | 120 | [(\<^const_syntax>\<open>String.Literal\<close>, K literal_tr'), | 
| 121 | (\<^const_syntax>\<open>String.empty_literal\<close>, K empty_literal_tr')]); | |
| 68028 | 122 | |
| 123 | end |