Theory UD

(* Title: UD/UD.thy
   Author: Mihails Milehins
   Copyright 2021 (C) Mihails Milehins

Infrastructure for unoverloading definitions.
*)

section‹UD›
theory UD
  imports "../CTR_Tools/CTR_Tools" Main
  keywords "ud" :: thy_decl
begin



subsection‹Import›

ML_file‹UD_With.ML›
ML_file‹UD_Consts.ML›
ML_file‹UD.ML›



subsectionud_with›

setupUD_With.UDWithData.setup

end