Theory SpecCheck.SpecCheck_Generators

✐‹creator "Kevin Kappelmann"›
section ‹Generators›
theory SpecCheck_Generators
imports SpecCheck_Base
begin

paragraph ‹Summary›
text ‹Generators for SpecCheck take a state and return a pair consisting of a generated value and
a new state. Refer to @{file "gen_base.ML"} for the most basic combinators.›

ML_file ‹gen_types.ML›
ML_file ‹gen_base.ML›
ML_file ‹gen_text.ML›
ML_file ‹gen_int.ML›
ML_file ‹gen_real.ML›
ML_file ‹gen_function.ML›
ML_file ‹gen_term.ML›
ML_file ‹gen.ML›

end