author | wenzelm |
Sat, 03 Sep 2005 16:50:22 +0200 | |
changeset 17244 | 0b2ff9541727 |
parent 7299 | 743b22579a2f |
child 22819 | a7b425bb668c |
permissions | -rw-r--r-- |
7299 | 1 |
|
17244 | 2 |
(* $Id$ *) |
3 |
||
4 |
theory MuIOA |
|
5 |
imports IOA MuckeSyn |
|
6 |
begin |
|
6471
08d12ef5fc19
added translation from IOA to mucalculus and corresponding modelchecker examples;
mueller
parents:
diff
changeset
|
7 |
|
08d12ef5fc19
added translation from IOA to mucalculus and corresponding modelchecker examples;
mueller
parents:
diff
changeset
|
8 |
consts |
17244 | 9 |
Internal_of_A :: "'a => bool" |
10 |
Internal_of_C :: "'a => bool" |
|
11 |
Start_of_A :: "'a => bool" |
|
12 |
Start_of_C :: "'a => bool" |
|
13 |
Trans_of_A :: "'a => 'b => bool" |
|
14 |
Trans_of_C :: "'a => 'b => bool" |
|
15 |
IntStep_of_A :: "'a => bool" |
|
16 |
IntStepStar_of_A :: "'a => bool" |
|
17 |
Move_of_A :: "'a => 'b => bool" |
|
18 |
isSimCA :: "'a => bool" |
|
6471
08d12ef5fc19
added translation from IOA to mucalculus and corresponding modelchecker examples;
mueller
parents:
diff
changeset
|
19 |
|
08d12ef5fc19
added translation from IOA to mucalculus and corresponding modelchecker examples;
mueller
parents:
diff
changeset
|
20 |
end |