diff -r a273bdac0934 -r 8b5f00202e1a src/HOL/MicroJava/J/State.thy --- a/src/HOL/MicroJava/J/State.thy Wed Oct 07 19:45:00 2015 +0200 +++ b/src/HOL/MicroJava/J/State.thy Wed Oct 07 23:28:49 2015 +0200 @@ -3,7 +3,7 @@ Copyright 1999 Technische Universitaet Muenchen *) -section {* Program State *} +section \Program State\ theory State imports TypeRel Value @@ -21,7 +21,7 @@ definition init_vars :: "('a \ ty) list => ('a \ val)" where "init_vars == map_of o map (\(n,T). (n,default_val T))" -type_synonym aheap = "loc \ obj" -- {* "@{text heap}" used in a translation below *} +type_synonym aheap = "loc \ obj" -- \"@{text heap}" used in a translation below\ type_synonym locals = "vname \ val" -- "simple state, i.e. variable contents" type_synonym state = "aheap \ locals" -- "heap, local parameter including This" @@ -52,7 +52,7 @@ definition raise_if :: "bool \ xcpt \ val option \ val option" where "raise_if b x xo \ if b \ (xo = None) then Some (Addr (XcptRef x)) else xo" -text {* Make @{text new_Addr} completely specified (at least for the code generator) *} +text \Make @{text new_Addr} completely specified (at least for the code generator)\ (* definition new_Addr :: "aheap => loc \ val option" where "new_Addr h \ SOME (a,x). (h a = None \ x = None) | x = Some (Addr (XcptRef OutOfMemory))" @@ -154,7 +154,7 @@ lemma c_hupd_fst [simp]: "fst (c_hupd h (x, s)) = x" by (simp add: c_hupd_def split_beta) -text {* Naive implementation for @{term "new_Addr"} by exhaustive search *} +text \Naive implementation for @{term "new_Addr"} by exhaustive search\ definition gen_new_Addr :: "aheap => nat \ loc \ val option" where "gen_new_Addr h n \