src/HOL/IMP/Com.thy
changeset 42174 d0be2722ce9f
parent 41589 bbd861837ebc
child 43141 11fce8564415
--- a/src/HOL/IMP/Com.thy	Wed Mar 30 22:53:18 2011 +0200
+++ b/src/HOL/IMP/Com.thy	Wed Mar 30 23:26:40 2011 +0200
@@ -11,11 +11,10 @@
   -- "an unspecified (arbitrary) type of locations 
       (adresses/names) for variables"
       
-types 
-  val   = nat -- "or anything else, @{text nat} used in examples"
-  state = "loc \<Rightarrow> val"
-  aexp  = "state \<Rightarrow> val"  
-  bexp  = "state \<Rightarrow> bool"
+type_synonym val = nat -- "or anything else, @{text nat} used in examples"
+type_synonym state = "loc \<Rightarrow> val"
+type_synonym aexp = "state \<Rightarrow> val"
+type_synonym bexp = "state \<Rightarrow> bool"
   -- "arithmetic and boolean expressions are not modelled explicitly here,"
   -- "they are just functions on states"