src/HOLCF/ex/Hoare.thy
changeset 25135 4f8176c940cf
parent 21404 eb85850d3eb7
child 25895 0eaadfa8889e
--- a/src/HOLCF/ex/Hoare.thy	Sun Oct 21 14:53:44 2007 +0200
+++ b/src/HOLCF/ex/Hoare.thy	Sun Oct 21 16:27:42 2007 +0200
@@ -24,9 +24,9 @@
 imports HOLCF
 begin
 
-consts
-  b1 :: "'a -> tr"
-  b2 :: "'a -> tr"
+axiomatization
+  b1 :: "'a -> tr" and
+  b2 :: "'a -> tr" and
   g :: "'a -> 'a"
 
 definition