|
3071
|
1 |
(* Title: HOLCF/IOA/meta_theory/CompoExecs.thy
|
|
3275
|
2 |
ID: $Id$
|
|
3071
|
3 |
Author: Olaf M"uller
|
|
|
4 |
Copyright 1996 TU Muenchen
|
|
|
5 |
|
|
|
6 |
Compositionality on Execution level.
|
|
|
7 |
*)
|
|
|
8 |
|
|
|
9 |
CompoExecs = Traces +
|
|
|
10 |
|
|
|
11 |
|
|
|
12 |
consts
|
|
|
13 |
|
|
|
14 |
ProjA ::"('a,'s * 't)execution => ('a,'s)execution"
|
|
|
15 |
ProjA2 ::"('a,'s * 't)pairs -> ('a,'s)pairs"
|
|
|
16 |
ProjB ::"('a,'s * 't)execution => ('a,'t)execution"
|
|
|
17 |
ProjB2 ::"('a,'s * 't)pairs -> ('a,'t)pairs"
|
|
|
18 |
Filter_ex ::"('a,'s)ioa => ('a,'s)execution => ('a,'s)execution"
|
|
|
19 |
Filter_ex2 ::"('a,'s)ioa => ('a,'s)pairs -> ('a,'s)pairs"
|
|
|
20 |
stutter ::"('a,'s)ioa => ('a,'s)execution => bool"
|
|
|
21 |
stutter2 ::"('a,'s)ioa => ('a,'s)pairs -> ('s => tr)"
|
|
|
22 |
|
|
|
23 |
|
|
|
24 |
defs
|
|
|
25 |
|
|
|
26 |
|
|
|
27 |
ProjA_def
|
|
|
28 |
"ProjA ex == (fst (fst ex), ProjA2`(snd ex))"
|
|
|
29 |
|
|
|
30 |
ProjB_def
|
|
|
31 |
"ProjB ex == (snd (fst ex), ProjB2`(snd ex))"
|
|
|
32 |
|
|
|
33 |
|
|
|
34 |
ProjA2_def
|
|
|
35 |
"ProjA2 == Map (%x.(fst x,fst(snd x)))"
|
|
|
36 |
|
|
|
37 |
ProjB2_def
|
|
|
38 |
"ProjB2 == Map (%x.(fst x,snd(snd x)))"
|
|
|
39 |
|
|
|
40 |
|
|
|
41 |
Filter_ex_def
|
|
|
42 |
"Filter_ex A ex == (fst ex,Filter_ex2 A`(snd ex))"
|
|
|
43 |
|
|
|
44 |
|
|
|
45 |
Filter_ex2_def
|
|
|
46 |
"Filter_ex2 A == Filter (%x.fst x:act A)"
|
|
|
47 |
|
|
|
48 |
stutter_def
|
|
|
49 |
"stutter A ex == ((stutter2 A`(snd ex)) (fst ex) ~= FF)"
|
|
|
50 |
|
|
|
51 |
stutter2_def
|
|
|
52 |
"stutter2 A ==(fix`(LAM h ex. (%s. case ex of
|
|
|
53 |
nil => TT
|
|
|
54 |
| x##xs => (flift1
|
|
|
55 |
(%p.(If Def ((fst p)~:act A)
|
|
|
56 |
then Def (s=(snd p))
|
|
|
57 |
else TT fi)
|
|
|
58 |
andalso (h`xs) (snd p))
|
|
|
59 |
`x)
|
|
|
60 |
)))"
|
|
|
61 |
|
|
|
62 |
|
|
|
63 |
|
|
|
64 |
|
|
|
65 |
end |