Theory ML_Unification.ML_Code_Utils

✐‹creator "Kevin Kappelmann"›
section ‹ML Code Utils›
theory ML_Code_Utils
  imports Pure
begin

paragraph ‹Summary›
text ‹Utilities to generate and manipulate (parsed) ML code.›

ML_file‹ml_code_util.ML›
ML_file‹ml_syntax_util.ML›

end