diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/NanoJava/Example.thy --- a/src/HOL/NanoJava/Example.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/NanoJava/Example.thy Fri Sep 20 19:51:08 2024 +0200 @@ -49,13 +49,13 @@ subsection "Program representation" axiomatization - N :: cname ("Nat") (* with mixfix because of clash with NatDef.Nat *) + N :: cname (\Nat\) (* with mixfix because of clash with NatDef.Nat *) and pred :: fname and suc add :: mname and any :: vname abbreviation - dummy :: expr ("<>") + dummy :: expr (\<>\) where "<> == LAcc any" abbreviation @@ -92,7 +92,7 @@ subsection "``atleast'' relation for interpretation of Nat ``values''" -primrec Nat_atleast :: "state \ val \ nat \ bool" ("_:_ \ _" [51, 51, 51] 50) where +primrec Nat_atleast :: "state \ val \ nat \ bool" (\_:_ \ _\ [51, 51, 51] 50) where "s:x\0 = (x\Null)" | "s:x\Suc n = (\a. x=Addr a \ heap s a \ None \ s:get_field s a pred\n)"