src/HOL/Bali/Bali.thy
author haftmann
Fri, 11 Jun 2010 17:14:02 +0200
changeset 37407 61dd8c145da7
parent 32634 9b19cbb0af28
permissions -rw-r--r--
declare lex_prod_def [code del]

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

header {* The Hoare logic for Bali. *}

theory Bali
imports AxExample AxSound AxCompl Trans
begin

end