src/HOLCF/IMP/HoareEx.thy
changeset 3664 2dced1ac2d8e
child 10835 f4745d77e620
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOLCF/IMP/HoareEx.thy	Tue Sep 09 12:09:06 1997 +0200
@@ -0,0 +1,18 @@
+(*  Title:      HOLCF/IMP/HoareEx.thy
+    ID:         $Id$
+    Author:     Tobias Nipkow, TUM
+    Copyright   1997 TUM
+
+An example from the HOLCF paper by Mueller, Nipkow, Oheimb, Slotosch.
+It demonstrates fixpoint reasoning by showing the correctness of the Hoare
+rule for while-loops.
+*)
+
+HoareEx = Denotational +
+
+types assn = state => bool
+
+constdefs hoare_valid :: [assn,com,assn] => bool ("|= {(1_)}/ (_)/ {(1_)}" 50)
+ "|= {A} c {B} == !s t. A s & D c `(Discr s) = Def t --> B t"
+
+end