src/HOL/UNITY/Simple/Reach.thy
changeset 42463 f270e3e18be5
parent 37936 1e4c5015a72e
child 44871 fbfdc5ac86be
--- a/src/HOL/UNITY/Simple/Reach.thy	Fri Apr 22 15:57:43 2011 +0200
+++ b/src/HOL/UNITY/Simple/Reach.thy	Sat Apr 23 13:00:19 2011 +0200
@@ -10,7 +10,7 @@
 
 typedecl vertex
 
-types    state = "vertex=>bool"
+type_synonym state = "vertex=>bool"
 
 consts
   init ::  "vertex"