Theory MFilter

section‹Presentation of All Variants as Studied in cite"C85" \label{sec:all}›

subsection‹Preliminaries: Modal Ultrafilter (Fig.~2 in cite"C85")›

theory MFilter imports HOML
begin 
text‹Some abbreviations for auxiliary operations.›
abbreviation a::"γ(γσ)σ" ("__") where "xS  S x"
abbreviation b::γ ("") where "  λx. "  
abbreviation c::γ ("U") where "U  λx. "
abbreviation d::"γγσ" ("__") where "φψ  x.((φ x)  (ψ x))"
abbreviation e::"γγγ" ("__") where "φψ  λx.((φ x)  (ψ x))"
abbreviation f::"γγ" ("¯_") where "¯ψ  λx. ¬(ψ x)"  

text‹Definition of modal filter.›
abbreviation g::"(γσ)σ" ("Filter") 
 where "Filter Φ  (((UΦ)  ¬(Φ))
          (φ ψ. (((φΦ)  (φψ))  (ψΦ))))
          (φ ψ. (((φΦ)  (ψΦ))  ((φψ)Φ)))"

text‹Definition of modal ultrafilter .›
abbreviation h::"(γσ)σ" ("UFilter") where 
 "UFilter Φ  (Filter Φ)(φ.((φΦ)  ((¯φ)Φ)))"

text‹Modal filter and modal ultrafilter are consistent.›
lemma "Φ φ.((UFilter Φ)  ¬((φΦ)  ((¯φ)Φ)))" by force
end