Theory Relation_Algebra_Models
section ‹Models of Relation Algebra›
theory Relation_Algebra_Models
imports Relation_Algebra Kleene_Algebra.Inf_Matrix
begin
text ‹We formalise two models. First we show the obvious: binary relations
form a relation algebra. Then we show that infinite matrices (which we
formalised originally for Kleene algebras) form models of relation algebra if
we restrict their element type to @{typ bool}.›
subsection ‹Binary Relations›
text ‹Since Isabelle's libraries for binary relations are very well
developed, the proof for this model is entirely trivial.›