Up to index of Isabelle/HOL/HoareParallel
theory RG_Syntaxheader {* \section{Concrete Syntax} *} theory RG_Syntax imports RG_Hoare Quote_Antiquote begin syntax "_Assign" :: "idt => 'b => 'a com" ("(´_ :=/ _)" [70, 65] 61) "_skip" :: "'a com" ("SKIP") "_Seq" :: "'a com => 'a com => 'a com" ("(_;;/ _)" [60,61] 60) "_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" \<rightharpoonup> "Basic «´ (_update_name x (λ_. a))»" "SKIP" \<rightleftharpoons> "Basic id" "c1;; c2" \<rightleftharpoons> "Seq c1 c2" "IF b THEN c1 ELSE c2 FI" \<rightharpoonup> "Cond .{b}. c1 c2" "IF b THEN c FI" \<rightleftharpoons> "IF b THEN c ELSE SKIP FI" "WHILE b DO c OD" \<rightharpoonup> "While .{b}. c" "AWAIT b THEN c END" \<rightleftharpoons> "Await .{b}. c" "〈c〉" \<rightleftharpoons> "AWAIT True THEN c END" "WAIT b END" \<rightleftharpoons> "AWAIT b THEN SKIP END" nonterminals prgs syntax "_PAR" :: "prgs => 'a" ("COBEGIN//_//COEND" 60) "_prg" :: "'a => prgs" ("_" 57) "_prgs" :: "['a, prgs] => prgs" ("_//\<parallel>//_" [60,57] 57) translations "_prg a" \<rightharpoonup> "[a]" "_prgs a ps" \<rightharpoonup> "a # ps" "_PAR ps" \<rightharpoonup> "ps" syntax "_prg_scheme" :: "['a, 'a, 'a, 'a] => prgs" ("SCHEME [_ ≤ _ < _] _" [0,0,0,60] 57) translations "_prg_scheme j i k c" \<rightleftharpoons> "(map (λi. c) [j..<k])" text {* Translations for variables before and after a transition: *} syntax "_before" :: "id => 'a" ("º_") "_after" :: "id => 'a" ("ª_") translations "ºx" \<rightleftharpoons> "x ´fst" "ªx" \<rightleftharpoons> "x ´snd" print_translation {* let fun quote_tr' f (t :: ts) = Term.list_comb (f $ Syntax.quote_tr' "_antiquote" t, ts) | quote_tr' _ _ = raise Match; val assert_tr' = quote_tr' (Syntax.const "_Assert"); fun bexp_tr' name ((Const ("Collect", _) $ t) :: ts) = quote_tr' (Syntax.const name) (t :: ts) | bexp_tr' _ _ = raise Match; fun upd_tr' (x_upd, T) = (case try (unsuffix RecordPackage.updateN) x_upd of SOME x => (x, if T = dummyT then T else Term.domain_type T) | NONE => raise Match); fun update_name_tr' (Free x) = Free (upd_tr' x) | update_name_tr' ((c as Const ("_free", _)) $ Free x) = c $ Free (upd_tr' x) | update_name_tr' (Const x) = Const (upd_tr' x) | update_name_tr' _ = raise Match; fun K_tr' (Abs (_,_,t)) = if null (loose_bnos t) then t else raise Match | K_tr' (Abs (_,_,Abs (_,_,t)$Bound 0)) = if null (loose_bnos t) then t else raise Match | K_tr' _ = raise Match; fun assign_tr' (Abs (x, _, f $ k $ Bound 0) :: ts) = quote_tr' (Syntax.const "_Assign" $ update_name_tr' f) (Abs (x, dummyT, K_tr' k) :: ts) | assign_tr' _ = raise Match; in [("Collect", assert_tr'), ("Basic", assign_tr'), ("Cond", bexp_tr' "_Cond"), ("While", bexp_tr' "_While_inv")] end *} end