equal
deleted
inserted
replaced
|
1 (* Title: HOL/IOA/example/Action.thy |
|
2 ID: $Id$ |
|
3 Author: Tobias Nipkow & Konrad Slind |
|
4 Copyright 1994 TU Muenchen |
|
5 |
|
6 The set of all actions of the system |
|
7 *) |
|
8 |
1 Action = Packet + |
9 Action = Packet + |
2 datatype 'm action = S_msg ('m) | R_msg ('m) |
10 datatype 'm action = S_msg ('m) | R_msg ('m) |
3 | S_pkt ('m packet) | R_pkt ('m packet) |
11 | S_pkt ('m packet) | R_pkt ('m packet) |
4 | S_ack (bool) | R_ack (bool) |
12 | S_ack (bool) | R_ack (bool) |
5 | C_m_s | C_m_r | C_r_s | C_r_r ('m) |
13 | C_m_s | C_m_r | C_r_s | C_r_r ('m) |