author | obua |
Sun, 09 May 2004 23:04:36 +0200 | |
changeset 14722 | 8e739a6eaf11 |
parent 11093 | 62c2e0af1d30 |
child 17479 | 68a7acb5f22e |
permissions | -rw-r--r-- |
7998 | 1 |
(* |
2 |
Properties of abstract class field |
|
3 |
$Id$ |
|
4 |
Author: Clemens Ballarin, started 15 November 1997 |
|
5 |
*) |
|
6 |
||
11093 | 7 |
Field = Factor + PID + |
7998 | 8 |
|
9 |
instance |
|
11093 | 10 |
field < domain (field_one_not_zero, field_integral) |
7998 | 11 |
|
12 |
instance |
|
13 |
field < factorial (TrueI, field_fact_prime) |
|
14 |
||
15 |
end |