Theory KAD.Modal_Kleene_Algebra_Models
section ‹Models of Modal Kleene Algebras›
theory Modal_Kleene_Algebra_Models
imports Kleene_Algebra.Kleene_Algebra_Models
Modal_Kleene_Algebra
begin
text ‹
This section develops the relation model. We also briefly develop the trace model for
antidomain Kleene algebras, but not for antirange or full modal Kleene algebras.
The reason is that traces are implemented as lists; we therefore expect tedious inductive
proofs in the presence of range. The language model is not particularly interesting.
›
definition rel_ad :: "'a rel ⇒ 'a rel" where
"rel_ad R = {(x,x) | x. ¬ (∃y. (x,y) ∈ R)}"