author | eberlm <eberlm@in.tum.de> |
Mon, 29 May 2017 09:14:15 +0200 | |
changeset 65956 | 639eb3617a86 |
parent 63167 | 0909deb8059b |
child 67613 | ce654b0e6d69 |
permissions | -rw-r--r-- |
4530 | 1 |
(* Title: HOL/IOA/Asig.thy |
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
2 |
Author: Tobias Nipkow & Konrad Slind |
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
3 |
Copyright 1994 TU Muenchen |
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
4 |
*) |
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
5 |
|
63167 | 6 |
section \<open>Action signatures\<close> |
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
7 |
|
17288 | 8 |
theory Asig |
9 |
imports Main |
|
10 |
begin |
|
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
11 |
|
62145 | 12 |
type_synonym 'a signature = "('a set * 'a set * 'a set)" |
13 |
||
14 |
definition "inputs" :: "'action signature => 'action set" |
|
15 |
where asig_inputs_def: "inputs == fst" |
|
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
16 |
|
62145 | 17 |
definition "outputs" :: "'action signature => 'action set" |
18 |
where asig_outputs_def: "outputs == (fst o snd)" |
|
17288 | 19 |
|
62145 | 20 |
definition "internals" :: "'action signature => 'action set" |
21 |
where asig_internals_def: "internals == (snd o snd)" |
|
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
22 |
|
62145 | 23 |
definition "actions" :: "'action signature => 'action set" |
24 |
where actions_def: "actions(asig) == (inputs(asig) Un outputs(asig) Un internals(asig))" |
|
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
25 |
|
62145 | 26 |
definition externals :: "'action signature => 'action set" |
27 |
where externals_def: "externals(asig) == (inputs(asig) Un outputs(asig))" |
|
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
28 |
|
62145 | 29 |
definition is_asig :: "'action signature => bool" |
30 |
where "is_asig(triple) == |
|
31 |
((inputs(triple) Int outputs(triple) = {}) & |
|
32 |
(outputs(triple) Int internals(triple) = {}) & |
|
33 |
(inputs(triple) Int internals(triple) = {}))" |
|
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
34 |
|
62145 | 35 |
definition mk_ext_asig :: "'action signature => 'action signature" |
36 |
where "mk_ext_asig(triple) == (inputs(triple), outputs(triple), {})" |
|
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
37 |
|
19801 | 38 |
|
39 |
lemmas asig_projections = asig_inputs_def asig_outputs_def asig_internals_def |
|
40 |
||
41 |
lemma int_and_ext_is_act: "[| a~:internals(S) ;a~:externals(S)|] ==> a~:actions(S)" |
|
42 |
apply (simp add: externals_def actions_def) |
|
43 |
done |
|
44 |
||
45 |
lemma ext_is_act: "[|a:externals(S)|] ==> a:actions(S)" |
|
46 |
apply (simp add: externals_def actions_def) |
|
47 |
done |
|
3078
984866a8f905
old IOA meta theory (see also new version in HOLCF/IOA/meta_theory);
mueller
parents:
diff
changeset
|
48 |
|
17288 | 49 |
end |