diff -r 4dc65845eab3 -r d8d7d1b785af src/HOL/MicroJava/J/Eval.thy --- a/src/HOL/MicroJava/J/Eval.thy Wed Feb 24 11:55:52 2010 +0100 +++ b/src/HOL/MicroJava/J/Eval.thy Mon Mar 01 13:40:23 2010 +0100 @@ -1,5 +1,4 @@ (* Title: HOL/MicroJava/J/Eval.thy - ID: $Id$ Author: David von Oheimb Copyright 1999 Technische Universitaet Muenchen *) @@ -11,22 +10,16 @@ -- "Auxiliary notions" -constdefs - fits :: "java_mb prog \ state \ val \ ty \ bool" ("_,_\_ fits _"[61,61,61,61]60) +definition fits :: "java_mb prog \ state \ val \ ty \ bool" ("_,_\_ fits _"[61,61,61,61]60) where "G,s\a' fits T \ case T of PrimT T' \ False | RefT T' \ a'=Null \ G\obj_ty(lookup_obj s a')\T" -constdefs - catch ::"java_mb prog \ xstate \ cname \ bool" ("_,_\catch _"[61,61,61]60) +definition catch :: "java_mb prog \ xstate \ cname \ bool" ("_,_\catch _"[61,61,61]60) where "G,s\catch C\ case abrupt s of None \ False | Some a \ G,store s\ a fits Class C" - - -constdefs - lupd :: "vname \ val \ state \ state" ("lupd'(_\_')"[10,10]1000) +definition lupd :: "vname \ val \ state \ state" ("lupd'(_\_')"[10,10]1000) where "lupd vn v \ \ (hp,loc). (hp, (loc(vn\v)))" -constdefs - new_xcpt_var :: "vname \ xstate \ xstate" +definition new_xcpt_var :: "vname \ xstate \ xstate" where "new_xcpt_var vn \ \(x,s). Norm (lupd(vn\the x) s)"