7998
|
1 |
(*
|
|
2 |
Ideals for commutative rings
|
|
3 |
$Id$
|
|
4 |
Author: Clemens Ballarin, started 24 September 1999
|
|
5 |
*)
|
|
6 |
|
17479
|
7 |
theory Ideal imports Ring begin
|
7998
|
8 |
|
|
9 |
consts
|
17479
|
10 |
ideal_of :: "('a::ring) set => 'a set"
|
|
11 |
is_ideal :: "('a::ring) set => bool"
|
|
12 |
is_pideal :: "('a::ring) set => bool"
|
7998
|
13 |
|
|
14 |
defs
|
17479
|
15 |
is_ideal_def: "is_ideal I == (ALL a: I. ALL b: I. a + b : I) &
|
|
16 |
(ALL a: I. - a : I) & 0 : I &
|
|
17 |
(ALL a: I. ALL r. a * r : I)"
|
|
18 |
ideal_of_def: "ideal_of S == Inter {I. is_ideal I & S <= I}"
|
|
19 |
is_pideal_def: "is_pideal I == (EX a. I = ideal_of {a})"
|
7998
|
20 |
|
17479
|
21 |
text {* Principle ideal domains *}
|
7998
|
22 |
|
17479
|
23 |
axclass pid < "domain"
|
|
24 |
pid_ax: "is_ideal I ==> is_pideal I"
|
7998
|
25 |
|
17479
|
26 |
end
|