changeset 62008 | cbedaddc9351 |
parent 62002 | f1599e98c4d0 |
child 62009 | ecb5212d5885 |
62007:3f8b97ceedb2 | 62008:cbedaddc9351 |
---|---|
3 *) |
3 *) |
4 |
4 |
5 section \<open>The (faulty) transmission channel (both directions)\<close> |
5 section \<open>The (faulty) transmission channel (both directions)\<close> |
6 |
6 |
7 theory Abschannel |
7 theory Abschannel |
8 imports "~~/src/HOL/HOLCF/IOA/meta_theory/IOA" Action |
8 imports "~~/src/HOL/HOLCF/IOA/IOA" Action |
9 begin |
9 begin |
10 |
10 |
11 datatype 'a abs_action = S 'a | R 'a |
11 datatype 'a abs_action = S 'a | R 'a |
12 |
12 |
13 definition |
13 definition |