src/HOL/Bali/Bali.thy
author blanchet
Thu, 16 Sep 2010 11:12:08 +0200
changeset 39452 70a57e40f795
parent 32634 9b19cbb0af28
permissions -rw-r--r--
factored out TSTP/SPASS/Vampire proof parsing; from "Sledgehammer_Reconstructo" to a new module "ATP_Proof"

(*  Author:     David von Oheimb
    Copyright   1999 Technische Universitaet Muenchen
*)

header {* The Hoare logic for Bali. *}

theory Bali
imports AxExample AxSound AxCompl Trans
begin

end