author | wenzelm |
Tue, 02 Jun 2015 09:10:05 +0200 | |
changeset 60357 | bc0827281dc1 |
parent 59189 | ad8e0a789af6 |
child 62390 | 842917225d56 |
permissions | -rw-r--r-- |
59189 | 1 |
section \<open>Concrete Syntax\<close> |
13020 | 2 |
|
15425 | 3 |
theory RG_Syntax |
4 |
imports RG_Hoare Quote_Antiquote |
|
5 |
begin |
|
13020 | 6 |
|
35107 | 7 |
abbreviation Skip :: "'a com" ("SKIP") |
8 |
where "SKIP \<equiv> Basic id" |
|
9 |
||
10 |
notation Seq ("(_;;/ _)" [60,61] 60) |
|
11 |
||
13020 | 12 |
syntax |
13 |
"_Assign" :: "idt \<Rightarrow> 'b \<Rightarrow> 'a com" ("(\<acute>_ :=/ _)" [70, 65] 61) |
|
14 |
"_Cond" :: "'a bexp \<Rightarrow> 'a com \<Rightarrow> 'a com \<Rightarrow> 'a com" ("(0IF _/ THEN _/ ELSE _/FI)" [0, 0, 0] 61) |
|
15 |
"_Cond2" :: "'a bexp \<Rightarrow> 'a com \<Rightarrow> 'a com" ("(0IF _ THEN _ FI)" [0,0] 56) |
|
16 |
"_While" :: "'a bexp \<Rightarrow> 'a com \<Rightarrow> 'a com" ("(0WHILE _ /DO _ /OD)" [0, 0] 61) |
|
17 |
"_Await" :: "'a bexp \<Rightarrow> 'a com \<Rightarrow> 'a com" ("(0AWAIT _ /THEN /_ /END)" [0,0] 61) |
|
18 |
"_Atom" :: "'a com \<Rightarrow> 'a com" ("(\<langle>_\<rangle>)" 61) |
|
19 |
"_Wait" :: "'a bexp \<Rightarrow> 'a com" ("(0WAIT _ END)" 61) |
|
20 |
||
21 |
translations |
|
35107 | 22 |
"\<acute>x := a" \<rightharpoonup> "CONST Basic \<guillemotleft>\<acute>(_update_name x (\<lambda>_. a))\<guillemotright>" |
53241 | 23 |
"IF b THEN c1 ELSE c2 FI" \<rightharpoonup> "CONST Cond \<lbrace>b\<rbrace> c1 c2" |
13020 | 24 |
"IF b THEN c FI" \<rightleftharpoons> "IF b THEN c ELSE SKIP FI" |
53241 | 25 |
"WHILE b DO c OD" \<rightharpoonup> "CONST While \<lbrace>b\<rbrace> c" |
26 |
"AWAIT b THEN c END" \<rightleftharpoons> "CONST Await \<lbrace>b\<rbrace> c" |
|
35113 | 27 |
"\<langle>c\<rangle>" \<rightleftharpoons> "AWAIT CONST True THEN c END" |
13020 | 28 |
"WAIT b END" \<rightleftharpoons> "AWAIT b THEN SKIP END" |
29 |
||
41229
d797baa3d57c
replaced command 'nonterminals' by slightly modernized version 'nonterminal';
wenzelm
parents:
35145
diff
changeset
|
30 |
nonterminal prgs |
13020 | 31 |
|
32 |
syntax |
|
33 |
"_PAR" :: "prgs \<Rightarrow> 'a" ("COBEGIN//_//COEND" 60) |
|
34 |
"_prg" :: "'a \<Rightarrow> prgs" ("_" 57) |
|
35 |
"_prgs" :: "['a, prgs] \<Rightarrow> prgs" ("_//\<parallel>//_" [60,57] 57) |
|
36 |
||
37 |
translations |
|
38 |
"_prg a" \<rightharpoonup> "[a]" |
|
39 |
"_prgs a ps" \<rightharpoonup> "a # ps" |
|
40 |
"_PAR ps" \<rightharpoonup> "ps" |
|
41 |
||
42 |
syntax |
|
43 |
"_prg_scheme" :: "['a, 'a, 'a, 'a] \<Rightarrow> prgs" ("SCHEME [_ \<le> _ < _] _" [0,0,0,60] 57) |
|
44 |
||
45 |
translations |
|
34940 | 46 |
"_prg_scheme j i k c" \<rightleftharpoons> "(CONST map (\<lambda>i. c) [j..<k])" |
13020 | 47 |
|
59189 | 48 |
text \<open>Translations for variables before and after a transition:\<close> |
13020 | 49 |
|
59189 | 50 |
syntax |
13020 | 51 |
"_before" :: "id \<Rightarrow> 'a" ("\<ordmasculine>_") |
52 |
"_after" :: "id \<Rightarrow> 'a" ("\<ordfeminine>_") |
|
59189 | 53 |
|
13020 | 54 |
translations |
35107 | 55 |
"\<ordmasculine>x" \<rightleftharpoons> "x \<acute>CONST fst" |
56 |
"\<ordfeminine>x" \<rightleftharpoons> "x \<acute>CONST snd" |
|
13020 | 57 |
|
59189 | 58 |
print_translation \<open> |
13020 | 59 |
let |
60 |
fun quote_tr' f (t :: ts) = |
|
42284 | 61 |
Term.list_comb (f $ Syntax_Trans.quote_tr' @{syntax_const "_antiquote"} t, ts) |
13020 | 62 |
| quote_tr' _ _ = raise Match; |
63 |
||
35113 | 64 |
val assert_tr' = quote_tr' (Syntax.const @{syntax_const "_Assert"}); |
13020 | 65 |
|
35107 | 66 |
fun bexp_tr' name ((Const (@{const_syntax Collect}, _) $ t) :: ts) = |
13020 | 67 |
quote_tr' (Syntax.const name) (t :: ts) |
68 |
| bexp_tr' _ _ = raise Match; |
|
69 |
||
25706 | 70 |
fun assign_tr' (Abs (x, _, f $ k $ Bound 0) :: ts) = |
42284 | 71 |
quote_tr' (Syntax.const @{syntax_const "_Assign"} $ Syntax_Trans.update_name_tr' f) |
72 |
(Abs (x, dummyT, Syntax_Trans.const_abs_tr' k) :: ts) |
|
13020 | 73 |
| assign_tr' _ = raise Match; |
74 |
in |
|
52143 | 75 |
[(@{const_syntax Collect}, K assert_tr'), |
76 |
(@{const_syntax Basic}, K assign_tr'), |
|
77 |
(@{const_syntax Cond}, K (bexp_tr' @{syntax_const "_Cond"})), |
|
78 |
(@{const_syntax While}, K (bexp_tr' @{syntax_const "_While"}))] |
|
13020 | 79 |
end |
59189 | 80 |
\<close> |
13020 | 81 |
|
82 |
end |