src/HOL/Bali/Bali.thy
author huffman
Mon, 26 Apr 2010 11:08:49 -0700
changeset 36367 49c7dee21a7f
parent 32634 9b19cbb0af28
permissions -rw-r--r--
fix another if-then-else parse error

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

header {* The Hoare logic for Bali. *}

theory Bali
imports AxExample AxSound AxCompl Trans
begin

end