src/HOL/NanoJava/State.thy
changeset 32960 69916a850301
parent 30235 58d147683393
child 35355 613e133966ea
child 35416 d8d7d1b785af
--- a/src/HOL/NanoJava/State.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/HOL/NanoJava/State.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      HOL/NanoJava/State.thy
-    ID:         $Id$
     Author:     David von Oheimb
     Copyright   2001 Technische Universitaet Muenchen
 *)
@@ -20,8 +19,8 @@
   = Null        --{* null reference *}
   | Addr loc    --{* address, i.e. location of object *}
 
-types	fields
-	= "(fname \<rightharpoonup> val)"
+types   fields
+        = "(fname \<rightharpoonup> val)"
 
         obj = "cname \<times> fields"
 
@@ -36,12 +35,12 @@
  "init_vars m == Option.map (\<lambda>T. Null) o m"
   
 text {* private: *}
-types	heap   = "loc   \<rightharpoonup> obj"
-        locals = "vname \<rightharpoonup> val"	
+types   heap   = "loc   \<rightharpoonup> obj"
+        locals = "vname \<rightharpoonup> val"  
 
 text {* private: *}
 record  state
-	= heap   :: heap
+        = heap   :: heap
           locals :: locals
 
 translations
@@ -97,7 +96,7 @@
   upd_obj    :: "loc => fname => val => state => state"
  "upd_obj a f v s \<equiv> let (C,fs) = the (heap s a) in hupd(a\<mapsto>(C,fs(f\<mapsto>v))) s"
 
-  new_Addr	:: "state => val"
+  new_Addr      :: "state => val"
  "new_Addr s == SOME v. (\<exists>a. v = Addr a \<and> (heap s) a = None) | v = Null"