Theory Monotonic_Boolean_Transformers_Instances
section ‹Instances of Monotonic Boolean Transformers›
theory Monotonic_Boolean_Transformers_Instances
imports Monotonic_Boolean_Transformers Pre_Post_Modal General_Refinement_Algebras
begin
sublocale mbt_algebra < mbta: bounded_idempotent_left_semiring
apply unfold_locales
apply (simp add: le_comp)
apply (simp add: sup_comp)
apply simp
apply simp
apply simp
apply simp
by (simp add: mult_assoc)
sublocale mbt_algebra < mbta_dual: bounded_idempotent_left_semiring where less = greater and less_eq = greater_eq and sup = inf and bot = top and top = bot
apply unfold_locales
using inf.bounded_iff inf_le1 inf_le2 mbta.mult_right_isotone apply simp
using inf_comp apply blast
apply simp
apply simp
apply simp
apply simp
by (simp add: mult_assoc)