Theory HOL_Syntax_Bundles

✐‹creator "Kevin Kappelmann"›
theory HOL_Syntax_Bundles
  imports
    HOL_Syntax_Bundles_Base
    HOL_Syntax_Bundles_Functions
    HOL_Syntax_Bundles_Groups
    HOL_Syntax_Bundles_Lattices
    HOL_Syntax_Bundles_Orders
    HOL_Syntax_Bundles_Relations
begin

paragraph ‹Summary›
text ‹Bundles to enable and disable syntax from HOL.›


end