diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Hoare_Parallel/RG_Syntax.thy --- a/src/HOL/Hoare_Parallel/RG_Syntax.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Hoare_Parallel/RG_Syntax.thy Fri Sep 20 19:51:08 2024 +0200 @@ -4,19 +4,19 @@ imports RG_Hoare Quote_Antiquote begin -abbreviation Skip :: "'a com" ("SKIP") +abbreviation Skip :: "'a com" (\SKIP\) where "SKIP \ Basic id" -notation Seq ("(_;;/ _)" [60,61] 60) +notation Seq (\(_;;/ _)\ [60,61] 60) syntax - "_Assign" :: "idt \ 'b \ 'a com" ("(\_ :=/ _)" [70, 65] 61) - "_Cond" :: "'a bexp \ 'a com \ 'a com \ 'a com" ("(0IF _/ THEN _/ ELSE _/FI)" [0, 0, 0] 61) - "_Cond2" :: "'a bexp \ 'a com \ 'a com" ("(0IF _ THEN _ FI)" [0,0] 56) - "_While" :: "'a bexp \ 'a com \ 'a com" ("(0WHILE _ /DO _ /OD)" [0, 0] 61) - "_Await" :: "'a bexp \ 'a com \ 'a com" ("(0AWAIT _ /THEN /_ /END)" [0,0] 61) - "_Atom" :: "'a com \ 'a com" ("(\_\)" 61) - "_Wait" :: "'a bexp \ 'a com" ("(0WAIT _ END)" 61) + "_Assign" :: "idt \ 'b \ 'a com" (\(\_ :=/ _)\ [70, 65] 61) + "_Cond" :: "'a bexp \ 'a com \ 'a com \ 'a com" (\(0IF _/ THEN _/ ELSE _/FI)\ [0, 0, 0] 61) + "_Cond2" :: "'a bexp \ 'a com \ 'a com" (\(0IF _ THEN _ FI)\ [0,0] 56) + "_While" :: "'a bexp \ 'a com \ 'a com" (\(0WHILE _ /DO _ /OD)\ [0, 0] 61) + "_Await" :: "'a bexp \ 'a com \ 'a com" (\(0AWAIT _ /THEN /_ /END)\ [0,0] 61) + "_Atom" :: "'a com \ 'a com" (\(\_\)\ 61) + "_Wait" :: "'a bexp \ 'a com" (\(0WAIT _ END)\ 61) translations "\x := a" \ "CONST Basic \\(_update_name x (\_. a))\" @@ -30,9 +30,9 @@ nonterminal prgs syntax - "_PAR" :: "prgs \ 'a" ("COBEGIN//_//COEND" 60) - "_prg" :: "'a \ prgs" ("_" 57) - "_prgs" :: "['a, prgs] \ prgs" ("_//\//_" [60,57] 57) + "_PAR" :: "prgs \ 'a" (\COBEGIN//_//COEND\ 60) + "_prg" :: "'a \ prgs" (\_\ 57) + "_prgs" :: "['a, prgs] \ prgs" (\_//\//_\ [60,57] 57) translations "_prg a" \ "[a]" @@ -40,7 +40,7 @@ "_PAR ps" \ "ps" syntax - "_prg_scheme" :: "['a, 'a, 'a, 'a] \ prgs" ("SCHEME [_ \ _ < _] _" [0,0,0,60] 57) + "_prg_scheme" :: "['a, 'a, 'a, 'a] \ prgs" (\SCHEME [_ \ _ < _] _\ [0,0,0,60] 57) translations "_prg_scheme j i k c" \ "(CONST map (\i. c) [j..Translations for variables before and after a transition:\ syntax - "_before" :: "id \ 'a" ("\_") - "_after" :: "id \ 'a" ("\_") + "_before" :: "id \ 'a" (\\_\) + "_after" :: "id \ 'a" (\\_\) translations "\x" \ "x \CONST fst"