author | oheimb |
Tue, 04 Jul 2000 10:54:46 +0200 | |
changeset 9241 | f961c1fdff50 |
parent 8029 | 05446a898852 |
child 12338 | de0f4a63baa5 |
permissions | -rw-r--r-- |
1476 | 1 |
(* Title: HOL/IMP/Com.thy |
924
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
2 |
ID: $Id$ |
1696 | 3 |
Author: Heiko Loetzbeyer & Robert Sandner & Tobias Nipkow, TUM |
924
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
4 |
Copyright 1994 TUM |
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
5 |
|
1696 | 6 |
Semantics of arithmetic and boolean expressions |
7 |
Syntax of commands |
|
924
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
8 |
*) |
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
9 |
|
8029 | 10 |
Com = Main + |
924
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
11 |
|
9241 | 12 |
types |
1696 | 13 |
loc |
9241 | 14 |
val = nat (* or anything else, nat used in examples *) |
15 |
state = loc => val |
|
16 |
aexp = state => val |
|
1696 | 17 |
bexp = state => bool |
924
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
18 |
|
9241 | 19 |
arities loc :: term |
924
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
20 |
|
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
21 |
datatype |
1696 | 22 |
com = SKIP |
9241 | 23 |
| ":==" loc aexp (infixl 60) |
1481 | 24 |
| Semi com com ("_; _" [60, 60] 10) |
25 |
| Cond bexp com com ("IF _ THEN _ ELSE _" 60) |
|
26 |
| While bexp com ("WHILE _ DO _" 60) |
|
924
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
27 |
|
806721cfbf46
new version of HOL/IMP with curried function application
clasohm
parents:
diff
changeset
|
28 |
end |