Theory Hoare
section ‹Hoare Logic›
theory Hoare
imports "HOL-Hoare.Hoare_Tac"
begin
subsection ‹Abstract syntax and semantics›
text ‹
The following abstract syntax and semantics of Hoare Logic over ▩‹WHILE›
programs closely follows the existing tradition in Isabelle/HOL of
formalizing the presentation given in \<^cite>‹‹\S6› in "Winskel:1993"›. See also
🗀‹~~/src/HOL/Hoare› and \<^cite>‹"Nipkow:1998:Winskel"›.
›
type_synonym 'a bexp = "'a set"
type_synonym 'a assn = "'a set"
type_synonym 'a var = "'a ⇒ nat"