(* Title: HOL/Hoare/Hoare_Logic.thy Author: Leonor Prensa Nieto & Tobias Nipkow Copyright 1998 TUM Author: Walter Guttmann (extension to total-correctness proofs) *) section ‹Hoare logic› theory Hoare_Logic imports Hoare_Syntax Hoare_Tac begin subsection ‹Sugared semantic embedding of Hoare logic› text ‹ Strictly speaking a shallow embedding (as implemented by Norbert Galm following Mike Gordon) would suffice. Maybe the datatype com comes in useful later. › type_synonym 'a bexp = "'a set" type_synonym 'a assn = "'a set"