Theory ML_IMap_Antiquotation

✐‹creator "Kevin Kappelmann"›
section ‹ML Indexed-Map Antiquotation›
theory ML_IMap_Antiquotation
  imports
    ML_Unification.ML_Functor_Instances
    ML_Unification.ML_General_Utils
begin

paragraph ‹Summary›
text ‹Antiquotation for indexed maps›

ML_file‹imap_antiquotation.ML›

MLfunctor_instancestruct_name: Standard_IMap_Antiquotation
  functor_name: IMap_Antiquotation
  id: ‹""›
  more_args: ‹val init_args = {
    sep = SOME "\n",
    encl = SOME ("", ""),
    encl_inner = SOME ("", ""),
    start = SOME 1,
    stop = SOME 2}›
local_setup Standard_IMap_Antiquotation.setup_attribute NONE
setup Standard_IMap_Antiquotation.setup_antiquotation

end