diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/IMPP/Natural.thy --- a/src/HOL/IMPP/Natural.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/IMPP/Natural.thy Fri Sep 20 19:51:08 2024 +0200 @@ -14,14 +14,14 @@ newlocs :: locals setlocs :: "state => locals => state" getlocs :: "state => locals" - update :: "state => vname => val => state" ("_/[_/::=/_]" [900,0,0] 900) + update :: "state => vname => val => state" (\_/[_/::=/_]\ [900,0,0] 900) abbreviation - loc :: "state => locals" ("_<_>" [75,0] 75) where + loc :: "state => locals" (\_<_>\ [75,0] 75) where "s == getlocs s X" inductive - evalc :: "[com,state, state] => bool" ("<_,_>/ -c-> _" [0,0, 51] 51) + evalc :: "[com,state, state] => bool" (\<_,_>/ -c-> _\ [0,0, 51] 51) where Skip: " -c-> s" @@ -52,7 +52,7 @@ [X::=s1]" inductive - evaln :: "[com,state,nat,state] => bool" ("<_,_>/ -_-> _" [0,0,0,51] 51) + evaln :: "[com,state,nat,state] => bool" (\<_,_>/ -_-> _\ [0,0,0,51] 51) where Skip: " -n-> s"