| author | clasohm |
| Mon, 05 Feb 1996 21:29:06 +0100 | |
| changeset 1476 | 608483c2122a |
| parent 1374 | 5e407f2a3323 |
| child 1625 | 40501958d0f6 |
| permissions | -rw-r--r-- |
| 1476 | 1 |
(* Title: HOL/Hoare/Examples.thy |
| 1335 | 2 |
ID: $Id$ |
| 1476 | 3 |
Author: Norbert Galm |
| 1335 | 4 |
Copyright 1995 TUM |
5 |
||
6 |
Various arithmetic examples. |
|
7 |
*) |
|
8 |
||
9 |
Examples = Hoare + Arith2 + |
|
10 |
||
11 |
syntax |
|
| 1476 | 12 |
"@1" :: nat ("1")
|
13 |
"@2" :: nat ("2")
|
|
| 1335 | 14 |
|
15 |
translations |
|
16 |
"1" == "Suc(0)" |
|
17 |
"2" == "Suc(Suc(0))" |
|
18 |
end |
|
19 |
||
20 |