Theory SpecCheck.SpecCheck_Show

✐‹creator "Kevin Kappelmann"›
section ‹Show›
theory SpecCheck_Show
imports Pure
begin

paragraph ‹Summary›
text ‹Show functions (pretty-printers) for SpecCheck take a value and return a @{ML_type Pretty.T}
representation of the value. Refer to @{file "show_base.ML"} for some basic examples.›

ML_file ‹show_types.ML›
ML_file ‹show_base.ML›
ML_file ‹show_term.ML›
ML_file ‹show.ML›

end