| author | wenzelm |
| Sun, 31 Jul 2016 17:25:38 +0200 | |
| changeset 63569 | 7e0b0db5e9ac |
| parent 63167 | 0909deb8059b |
| child 65897 | 94b0da1b242e |
| permissions | -rw-r--r-- |
(* Author: Florian Haftmann, TU Muenchen *) section \<open>Pervasive test of code generator\<close> theory Generate imports Candidates "~~/src/HOL/Library/AList_Mapping" "~~/src/HOL/Library/Finite_Lattice" begin text \<open> If any of the checks fails, inspect the code generated by a corresponding \<open>export_code\<close> command. \<close> export_code _ checking SML OCaml? Haskell? Scala end