equal
deleted
inserted
replaced
1 (* Title: HOL/HOLCF/IOA/ABP/Receiver.thy |
1 (* Title: HOL/HOLCF/IOA/ABP/Receiver.thy |
2 Author: Olaf Müller |
2 Author: Olaf Müller |
3 *) |
3 *) |
4 |
4 |
5 section {* The implementation: receiver *} |
5 section \<open>The implementation: receiver\<close> |
6 |
6 |
7 theory Receiver |
7 theory Receiver |
8 imports "~~/src/HOL/HOLCF/IOA/meta_theory/IOA" Action Lemmas |
8 imports "~~/src/HOL/HOLCF/IOA/meta_theory/IOA" Action Lemmas |
9 begin |
9 begin |
10 |
10 |
11 type_synonym |
11 type_synonym |
12 'm receiver_state = "'m list * bool" -- {* messages, mode *} |
12 'm receiver_state = "'m list * bool" \<comment> \<open>messages, mode\<close> |
13 |
13 |
14 definition |
14 definition |
15 rq :: "'m receiver_state => 'm list" where |
15 rq :: "'m receiver_state => 'm list" where |
16 "rq = fst" |
16 "rq = fst" |
17 |
17 |