src/HOL/Bali/Bali.thy
author wenzelm
Wed, 01 Sep 2010 17:59:06 +0200
changeset 38975 ef13a2cc97be
parent 32634 9b19cbb0af28
permissions -rw-r--r--
actually declare "_constrainAbs" as @{syntax_const};

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

header {* The Hoare logic for Bali. *}

theory Bali
imports AxExample AxSound AxCompl Trans
begin

end