added filter for Boogie verification conditions (to prune assertions already proved by Boogie/Z3)
(* Author: David von Oheimb
Copyright 1999 Technische Universitaet Muenchen
*)
header {* The Hoare logic for Bali. *}
theory Bali
imports AxExample AxSound AxCompl Trans
begin
end