Theory Orders

✐‹creator "Kevin Kappelmann"›
section ‹Orders›
theory Orders
  imports
    Equivalence_Relations
    Linear_Orders
    Order_Functions
    Order_Functors
    Partial_Equivalence_Relations
    Partial_Orders
    Preorders
begin

paragraph ‹Summary›
text ‹Basic order-theoretic concepts.›


end