src/HOL/Induct/Com.thy
changeset 41818 6d4c3ee8219d
parent 36862 952b2b102a0a
child 44174 d1d79f0e1ea6
--- a/src/HOL/Induct/Com.thy	Tue Feb 22 16:47:18 2011 +0100
+++ b/src/HOL/Induct/Com.thy	Tue Feb 22 17:06:14 2011 +0100
@@ -10,7 +10,7 @@
 theory Com imports Main begin
 
 typedecl loc
-types  state = "loc => nat"
+type_synonym state = "loc => nat"
 
 datatype
   exp = N nat