diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/IMP/OO.thy --- a/src/HOL/IMP/OO.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/IMP/OO.thy Fri Sep 20 19:51:08 2024 +0200 @@ -4,7 +4,7 @@ (* FIXME: move to HOL/Fun *) abbreviation fun_upd2 :: "('a \ 'b \ 'c) \ 'a \ 'b \ 'c \ 'a \ 'b \ 'c" - ("_/'((2_,_ :=/ _)')" [1000,0,0,0] 900) + (\_/'((2_,_ :=/ _)')\ [1000,0,0,0] 900) where "f(x,y := z) == f(x := (f x)(y := z))" type_synonym addr = nat @@ -18,12 +18,12 @@ Null | New | V string | - Faccess exp string ("_\/_" [63,1000] 63) | - Vassign string exp ("(_ ::=/ _)" [1000,61] 62) | - Fassign exp string exp ("(_\_ ::=/ _)" [63,0,62] 62) | - Mcall exp string exp ("(_\/_<_>)" [63,0,0] 63) | - Seq exp exp ("_;/ _" [61,60] 60) | - If bexp exp exp ("IF _/ THEN (2_)/ ELSE (2_)" [0,0,61] 61) + Faccess exp string (\_\/_\ [63,1000] 63) | + Vassign string exp (\(_ ::=/ _)\ [1000,61] 62) | + Fassign exp string exp (\(_\_ ::=/ _)\ [63,0,62] 62) | + Mcall exp string exp (\(_\/_<_>)\ [63,0,0] 63) | + Seq exp exp (\_;/ _\ [61,60] 60) | + If bexp exp exp (\IF _/ THEN (2_)/ ELSE (2_)\ [0,0,61] 61) and bexp = B bool | Not bexp | And bexp bexp | Eq exp exp type_synonym menv = "string \ exp" @@ -31,9 +31,9 @@ inductive big_step :: "menv \ exp \ config \ ref \ config \ bool" - ("(_ \/ (_/ \ _))" [60,0,60] 55) and + (\(_ \/ (_/ \ _))\ [60,0,60] 55) and bval :: "menv \ bexp \ config \ bool \ config \ bool" - ("_ \ _ \ _" [60,0,60] 55) + (\_ \ _ \ _\ [60,0,60] 55) where Null: "me \ (Null,c) \ (null,c)" |