diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Induct/Com.thy --- a/src/HOL/Induct/Com.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Induct/Com.thy Fri Sep 20 19:51:08 2024 +0200 @@ -16,13 +16,13 @@ exp = N nat | X loc | Op "nat => nat => nat" exp exp - | valOf com exp ("VALOF _ RESULTIS _" 60) + | valOf com exp (\VALOF _ RESULTIS _\ 60) and com = SKIP - | Assign loc exp (infixl ":=" 60) - | Semi com com ("_;;_" [60, 60] 60) - | Cond exp com com ("IF _ THEN _ ELSE _" 60) - | While exp com ("WHILE _ DO _" 60) + | Assign loc exp (infixl \:=\ 60) + | Semi com com (\_;;_\ [60, 60] 60) + | Cond exp com com (\IF _ THEN _ ELSE _\ 60) + | While exp com (\WHILE _ DO _\ 60) subsection \Commands\ @@ -30,7 +30,7 @@ text\Execution of commands\ abbreviation (input) - generic_rel ("_/ -|[_]-> _" [50,0,50] 50) where + generic_rel (\_/ -|[_]-> _\ [50,0,50] 50) where "esig -|[eval]-> ns == (esig,ns) \ eval" text\Command execution. Natural numbers represent Booleans: 0=True, 1=False\ @@ -38,7 +38,7 @@ inductive_set exec :: "((exp*state) * (nat*state)) set => ((com*state)*state)set" and exec_rel :: "com * state => ((exp*state) * (nat*state)) set => state => bool" - ("_/ -[_]-> _" [50,0,50] 50) + (\_/ -[_]-> _\ [50,0,50] 50) for eval :: "((exp*state) * (nat*state)) set" where "csig -[eval]-> s == (csig,s) \ exec eval" @@ -108,7 +108,7 @@ inductive_set eval :: "((exp*state) * (nat*state)) set" - and eval_rel :: "[exp*state,nat*state] => bool" (infixl "-|->" 50) + and eval_rel :: "[exp*state,nat*state] => bool" (infixl \-|->\ 50) where "esig -|-> ns == (esig, ns) \ eval"