Theory Linear_Aggregation_Algebras
section ‹Algebras for Aggregation and Minimisation with a Linear Order›
text ‹
This theory gives several classes of instances of linear aggregation lattices as described in \<^cite>‹"Guttmann2018a"›.
Each of these instances can be used as edge weights and the resulting graphs will form s-algebras and m-algebras as shown in a separate theory.
›
theory Linear_Aggregation_Algebras
imports Matrix_Aggregation_Algebras HOL.Real
begin
no_notation
inf (infixl "⊓" 70)
and uminus ("- _" [81] 80)
subsection ‹Linearly Ordered Commutative Semigroups›
text ‹
Any linearly ordered commutative semigroup extended by new least and greatest elements forms a linear aggregation lattice.
The extension is done so that the new least element is a unit of aggregation and the new greatest element is a zero of aggregation.
›