src/HOL/Predicate_Compile_Examples/Examples.thy
changeset 42463 f270e3e18be5
parent 42208 02513eb26eb7
child 45970 b6d0cff57d96
--- a/src/HOL/Predicate_Compile_Examples/Examples.thy	Fri Apr 22 15:57:43 2011 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Examples.thy	Sat Apr 23 13:00:19 2011 +0200
@@ -16,7 +16,7 @@
                             
 datatype ('nts,'ts) rule = rule 'nts "('nts,'ts) symbol list"
 
-types ('nts,'ts) grammar = "('nts,'ts) rule set * 'nts"
+type_synonym ('nts,'ts) grammar = "('nts,'ts) rule set * 'nts"
 
 fun rules :: "('nts,'ts) grammar => ('nts,'ts) rule set"
 where
@@ -120,9 +120,8 @@
 
 subsection {* IMP *}
 
-types
-  var = nat
-  state = "int list"
+type_synonym var = nat
+type_synonym state = "int list"
 
 datatype com =
   Skip |
@@ -217,10 +216,9 @@
 
 text {* thanks to Elke Salecker *}
 
-types
-  vname = nat
-  vvalue = int
-  var_assign = "vname \<Rightarrow> vvalue"  --"variable assignment"
+type_synonym vname = nat
+type_synonym vvalue = int
+type_synonym var_assign = "vname \<Rightarrow> vvalue"  --"variable assignment"
 
 datatype ir_expr = 
   IrConst vvalue
@@ -248,9 +246,8 @@
 
 subsection {* Another semantics *}
 
-types
-  name = nat --"For simplicity in examples"
-  state' = "name \<Rightarrow> nat"
+type_synonym name = nat --"For simplicity in examples"
+type_synonym state' = "name \<Rightarrow> nat"
 
 datatype aexp = N nat | V name | Plus aexp aexp