author | clasohm |
Fri, 24 Nov 1995 11:46:23 +0100 | |
changeset 1367 | 78bdb2d04771 |
parent 1274 | ea0668a1c0ba |
child 1479 | 21eb5e156d91 |
permissions | -rw-r--r-- |
1274 | 1 |
(* Title: HOLCF/ex/Fix2.thy |
2 |
ID: $Id$ |
|
3 |
Author: Franz Regensburger |
|
4 |
Copyright 1995 Technische Universitaet Muenchen |
|
5 |
||
6 |
Show that fix is the unique least fixed-point operator. |
|
7 |
From axioms gix1_def,gix2_def it follows that fix = gix |
|
8 |
||
9 |
*) |
|
10 |
||
11 |
Fix2 = Fix + |
|
12 |
||
13 |
consts |
|
14 |
||
15 |
gix :: "('a->'a)->'a" |
|
16 |
||
17 |
rules |
|
18 |
||
19 |
gix1_def "F`(gix`F) = gix`F" |
|
20 |
gix2_def "F`y=y ==> gix`F << y" |
|
21 |
||
22 |
end |
|
23 |
||
24 |
||
25 |
||
26 |
||
27 |
||
28 |
||
29 |
||
30 |
||
31 |
||
32 |
||
33 |
||
34 |
||
35 |
||
36 |
||
37 |
||
38 |