src/HOL/MicroJava/BV/JVMType.thy
changeset 42463 f270e3e18be5
parent 42150 b0c0638c4aad
child 47994 d7c0aa802f0d
--- a/src/HOL/MicroJava/BV/JVMType.thy	Fri Apr 22 15:57:43 2011 +0200
+++ b/src/HOL/MicroJava/BV/JVMType.thy	Sat Apr 23 13:00:19 2011 +0200
@@ -9,14 +9,13 @@
 imports JType
 begin
 
-types
-  locvars_type = "ty err list"
-  opstack_type = "ty list"
-  state_type   = "opstack_type \<times> locvars_type"
-  state        = "state_type option err"    -- "for Kildall"
-  method_type  = "state_type option list"   -- "for BVSpec"
-  class_type   = "sig \<Rightarrow> method_type"
-  prog_type    = "cname \<Rightarrow> class_type"
+type_synonym locvars_type = "ty err list"
+type_synonym opstack_type = "ty list"
+type_synonym state_type = "opstack_type \<times> locvars_type"
+type_synonym state = "state_type option err"    -- "for Kildall"
+type_synonym method_type = "state_type option list"   -- "for BVSpec"
+type_synonym class_type = "sig \<Rightarrow> method_type"
+type_synonym prog_type = "cname \<Rightarrow> class_type"
 
 
 definition stk_esl :: "'c prog \<Rightarrow> nat \<Rightarrow> ty list esl" where