Theory utp_theory
section ‹ UTP Theories ›
theory utp_theory
imports utp_rel_laws
begin
text ‹ Here, we mechanise a representation of UTP theories using locales~\<^cite>‹"Ballarin06"›. We also
link them to the HOL-Algebra library~\<^cite>‹"Ballarin17"›, which allows us to import properties from
complete lattices and Galois connections. ›
subsection ‹ Complete lattice of predicates ›
definition upred_lattice :: "('α upred) gorder" (‹𝒫›) where
"upred_lattice = ⦇ carrier = UNIV, eq = (=), le = (⊑) ⦈"
text ‹ @{term "𝒫"} is the complete lattice of alphabetised predicates. All other theories will
be defined relative to it. ›