author | paulson <lp15@cam.ac.uk> |
Tue, 02 May 2023 12:51:05 +0100 | |
changeset 77934 | 01c88cf514fc |
parent 75647 | 34cd1d210b92 |
permissions | -rw-r--r-- |
75647 | 1 |
|
2 |
(* Author: Florian Haftmann, TU Muenchen *) |
|
3 |
||
4 |
section \<open>Pervasive test of code generator\<close> |
|
5 |
||
6 |
theory Generate_Abstract_Char |
|
7 |
imports |
|
8 |
Candidates |
|
9 |
"HOL-Library.Code_Abstract_Char" |
|
10 |
begin |
|
11 |
||
12 |
text \<open> |
|
13 |
If any of the checks fails, inspect the code generated |
|
14 |
by a corresponding \<open>export_code\<close> command. |
|
15 |
\<close> |
|
16 |
||
17 |
export_code _ checking SML OCaml? Haskell? Scala |
|
18 |
||
19 |
end |