src/HOL/NanoJava/State.thy
changeset 11499 7a7bb59a05db
parent 11497 0e66e0114d9a
child 11507 4b32a46ffd29
--- a/src/HOL/NanoJava/State.thy	Thu Aug 09 22:07:39 2001 +0200
+++ b/src/HOL/NanoJava/State.thy	Thu Aug 09 23:42:45 2001 +0200
@@ -15,7 +15,6 @@
 
 text {* locations, i.e.\ abstract references to objects *}
 typedecl loc 
-arities  loc :: "term"
 
 datatype val
   = Null        (* null reference *)