Theory HS_VC_MKA_rel
subsection ‹Verification of hybrid programs›
text ‹ We show that relations form an antidomain Kleene algebra. This allows us to inherit
the rules of the wlp calculus for regular programs. Finally, we derive three methods for
verifying correctness specifications for the continuous dynamics of hybrid systems in this
setting. ›
theory HS_VC_MKA_rel
imports
"../HS_ODEs"
"HS_VC_MKA"
"../HS_VC_KA_rel"
begin
definition rel_ad :: "'a rel ⇒ 'a rel" where
"rel_ad R = {(x,x) | x. ¬ (∃y. (x,y) ∈ R)}"