| author | lcp |
| Tue, 25 Jul 1995 17:31:53 +0200 | |
| changeset 1196 | d43c1f7a53fe |
| parent 1155 | 928a16e02f9f |
| child 1200 | d4551b1a6da7 |
| permissions | -rw-r--r-- |
| 1123 | 1 |
(* Title: ZF/AC/first.thy |
2 |
ID: $Id$ |
|
3 |
Author: Krzysztof Gr`abczewski |
|
4 |
||
5 |
Theory helpful in proofs using first element of a well ordered set |
|
6 |
*) |
|
7 |
||
8 |
first = Order + |
|
9 |
||
10 |
consts |
|
11 |
||
12 |
first :: "[i, i, i] => o" |
|
13 |
||
14 |
defs |
|
15 |
||
| 1196 | 16 |
first_def "first(u, X, R) |
17 |
== u:X & (ALL v:X. v~=u --> <u,v> : R)" |
|
| 1123 | 18 |
|
19 |
end |