# HG changeset patch # User wenzelm # Date 1082984178 -7200 # Node ID 3506a9af46fc85577a7af7eb677e66f51d26ab44 # Parent 3d760a971fde80cdd81f736acedcf1072cc08d6b *** empty log message *** diff -r 3d760a971fde -r 3506a9af46fc src/HOL/Bali/Conform.thy --- a/src/HOL/Bali/Conform.thy Mon Apr 26 14:54:45 2004 +0200 +++ b/src/HOL/Bali/Conform.thy Mon Apr 26 14:56:18 2004 +0200 @@ -26,7 +26,7 @@ constdefs - gext :: "st \ st \ bool"    ("_\|_"    [71,71] 70) + gext :: "st \ st \ bool" ("_\|_" [71,71] 70) "s\|s' \ \r. \obj\globs s r: \obj'\globs s' r: tag obj'= tag obj" text {* For the the proof of type soundness we will need the @@ -186,7 +186,7 @@ constdefs lconf :: "prog \ st \ ('a, val) table \ ('a, ty) table \ bool" - ("_,_\_[\\]_" [71,71,71,71] 70) + ("_,_\_[\\]_" [71,71,71,71] 70) "G,s\vs[\\]Ts \ \n. \T\Ts n: \v\vs n: G,s\v\\T" lemma lconfD: "\G,s\vs[\\]Ts; Ts n = Some T\ \ G,s\(the (vs n))\\T" @@ -272,7 +272,7 @@ constdefs wlconf :: "prog \ st \ ('a, val) table \ ('a, ty) table \ bool" - ("_,_\_[\\\]_" [71,71,71,71] 70) + ("_,_\_[\\\]_" [71,71,71,71] 70) "G,s\vs[\\\]Ts \ \n. \T\Ts n: \ v\vs n: G,s\v\\T" lemma wlconfD: "\G,s\vs[\\\]Ts; Ts n = Some T; vs n = Some v\ \ G,s\v\\T" @@ -389,7 +389,7 @@ constdefs - conforms :: "state \ env_ \ bool"  (  "_\\_" [71,71] 70) + conforms :: "state \ env_ \ bool" ( "_\\_" [71,71] 70) "xs\\E \ let (G, L) = E; s = snd xs; l = locals s in (\r. \obj\globs s r: G,s\obj \\\r) \ \ G,s\l [\\\]L\ \ diff -r 3d760a971fde -r 3506a9af46fc src/HOL/Bali/Decl.thy --- a/src/HOL/Bali/Decl.thy Mon Apr 26 14:54:45 2004 +0200 +++ b/src/HOL/Bali/Decl.thy Mon Apr 26 14:56:18 2004 +0200 @@ -366,9 +366,9 @@ consts - Object_mdecls ::  "mdecl list" --{* methods of Object *} - SXcpt_mdecls ::  "mdecl list" --{* methods of SXcpts *} - ObjectC ::  "cdecl" --{* declaration of root class *} + Object_mdecls :: "mdecl list" --{* methods of Object *} + SXcpt_mdecls :: "mdecl list" --{* methods of SXcpts *} + ObjectC :: "cdecl" --{* declaration of root class *} SXcptC ::"xname \ cdecl" --{* declarations of throwable classes *} defs diff -r 3d760a971fde -r 3506a9af46fc src/HOL/Bali/Evaln.thy --- a/src/HOL/Bali/Evaln.thy Mon Apr 26 14:54:45 2004 +0200 +++ b/src/HOL/Bali/Evaln.thy Mon Apr 26 14:56:18 2004 +0200 @@ -57,7 +57,7 @@ evalsn:: "[prog, state, expr list, val list, nat, state] \ bool" ("_\_ \_\\_\_\ _" [61,61,61,61,61,61] 60) execn :: "[prog, state, stmt , nat, state] \ bool" - ("_\_ \_\_\ _"   [61,61,65, 61,61] 60) + ("_\_ \_\_\ _" [61,61,65, 61,61] 60) translations diff -r 3d760a971fde -r 3506a9af46fc src/HOL/Bali/TypeRel.thy --- a/src/HOL/Bali/TypeRel.thy Mon Apr 26 14:54:45 2004 +0200 +++ b/src/HOL/Bali/TypeRel.thy Mon Apr 26 14:56:18 2004 +0200 @@ -29,16 +29,16 @@ consts -(*subint1, in Decl.thy*)  (* direct subinterface *) -(*subint , by translation*)   (* subinterface (+ identity) *) -(*subcls1, in Decl.thy*)  (* direct subclass *) -(*subcls , by translation*)   (* subclass *) -(*subclseq, by translation*)  (* subclass + identity *) +(*subint1, in Decl.thy*) (* direct subinterface *) +(*subint , by translation*) (* subinterface (+ identity) *) +(*subcls1, in Decl.thy*) (* direct subclass *) +(*subcls , by translation*) (* subclass *) +(*subclseq, by translation*) (* subclass + identity *) implmt1 :: "prog \ (qtname \ qtname) set" --{* direct implementation *} - implmt :: "prog \ (qtname \ qtname) set" --{* implementation *} + implmt :: "prog \ (qtname \ qtname) set" --{* implementation *} widen :: "prog \ (ty \ ty ) set" --{* widening *} narrow :: "prog \ (ty \ ty ) set" --{* narrowing *} - cast :: "prog \ (ty \ ty ) set"  --{* casting *} + cast :: "prog \ (ty \ ty ) set" --{* casting *} syntax