Theory Generate_Abstract_Char


(* Author: Florian Haftmann, TU Muenchen *)

section ‹Pervasive test of code generator›

theory Generate_Abstract_Char
imports
  Candidates
  "HOL-Library.Code_Abstract_Char"
begin

text ‹
  If any of the checks fails, inspect the code generated
  by a corresponding export_code› command.
›

export_code _ checking SML OCaml? Haskell? Scala

end