1050
|
1 |
(* Title: HOL/IOA/ABP/Impl_finite.thy
|
|
2 |
ID: $Id$
|
|
3 |
Author: Tobias Nipkow & Olaf Mueller
|
|
4 |
Copyright 1995 TU Muenchen
|
|
5 |
|
|
6 |
The finite implementation
|
|
7 |
*)
|
|
8 |
|
|
9 |
Impl_finite = Sender + Receiver + Abschannel_finite +
|
|
10 |
|
|
11 |
types
|
|
12 |
|
|
13 |
'm impl_fin_state
|
|
14 |
= "'m sender_state * 'm receiver_state * 'm packet list * bool list"
|
|
15 |
(* sender_state * receiver_state * srch_state * rsch_state *)
|
|
16 |
|
|
17 |
consts
|
|
18 |
|
|
19 |
impl_fin_ioa :: "('m action, 'm impl_fin_state)ioa"
|
|
20 |
sen_fin :: "'m impl_fin_state => 'm sender_state"
|
|
21 |
rec_fin :: "'m impl_fin_state => 'm receiver_state"
|
|
22 |
srch_fin :: "'m impl_fin_state => 'm packet list"
|
|
23 |
rsch_fin :: "'m impl_fin_state => bool list"
|
|
24 |
|
|
25 |
defs
|
|
26 |
|
|
27 |
impl_fin_def
|
|
28 |
"impl_fin_ioa == (sender_ioa || receiver_ioa || srch_fin_ioa || rsch_fin_ioa)"
|
|
29 |
sen_fin_def "sen_fin == fst"
|
|
30 |
rec_fin_def "rec_fin == fst o snd"
|
|
31 |
srch_fin_def "srch_fin == fst o snd o snd"
|
|
32 |
rsch_fin_def "rsch_fin == snd o snd o snd"
|
|
33 |
|
|
34 |
end
|
|
35 |
|