Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit b5440be

Browse files
committed
feat(ring_theory/noetherian): is_noetherian_ring_range
1 parent 8e381f6 commit b5440be

File tree

1 file changed

+7
-0
lines changed

1 file changed

+7
-0
lines changed

src/ring_theory/noetherian.lean

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -8,6 +8,7 @@ import data.equiv.algebra
88
import data.polynomial
99
import linear_algebra.linear_combination
1010
import ring_theory.ideal_operations
11+
import ring_theory.subring
1112

1213
open set lattice
1314

@@ -305,6 +306,12 @@ begin
305306
convert order_embedding.well_founded (order_embedding.rsymm (ideal.lt_order_embedding_of_surjective f hf)) H
306307
end
307308

309+
theorem is_noetherian_ring_range {R} [comm_ring R] {S} [comm_ring S] (f : R → S) (hf : is_ring_hom f)
310+
(h : is_noetherian_ring R) : is_noetherian_ring (set.range f) :=
311+
is_noetherian_ring_of_surjective _ _ (λ r, ⟨f r, r, rfl⟩)
312+
⟨subtype.eq $ is_ring_hom.map_one f, λ x y, subtype.eq $ is_ring_hom.map_mul f, λ x y, subtype.eq $ is_ring_hom.map_add f⟩
313+
(λ ⟨y, r, h⟩, ⟨r, subtype.eq h⟩) h
314+
308315
theorem is_noetherian_ring_of_ring_equiv (R) [comm_ring R] {S} [comm_ring S]
309316
(f : R ≃r S) (H : is_noetherian_ring R) : is_noetherian_ring S :=
310317
is_noetherian_ring_of_surjective R S f.1 f.2 f.1.bijective.2 H

0 commit comments

Comments
 (0)