src/HOL/IMPP/Hoare.thy
changeset 42174 d0be2722ce9f
parent 41529 ba60efa2fd08
child 42793 88bee9f6eec7
--- a/src/HOL/IMPP/Hoare.thy	Wed Mar 30 22:53:18 2011 +0200
+++ b/src/HOL/IMPP/Hoare.thy	Wed Mar 30 23:26:40 2011 +0200
@@ -16,7 +16,7 @@
   vs. simultaneous recursion in call rule
 *}
 
-types 'a assn = "'a => state => bool"
+type_synonym 'a assn = "'a => state => bool"
 translations
   (type) "'a assn" <= (type) "'a => state => bool"