adding values to show and ensure that values works with complex terms and restores numerals on natural numbers
header {* Install quickcheck of SML code generator *}
theory SML_Quickcheck
imports Main
begin
setup {*
Inductive_Codegen.quickcheck_setup #>
Context.theory_map (Quickcheck.add_generator ("SML", Codegen.test_term))
*}
end