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

Commit 8d8c356

Browse files
committed
chore(ring_theory/noetherian): add fg_span and fg_span_singleton (#6709)
1 parent f221bfd commit 8d8c356

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

src/ring_theory/noetherian.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -109,6 +109,12 @@ end
109109
theorem fg_bot : (⊥ : submodule R M).fg :=
110110
⟨∅, by rw [finset.coe_empty, span_empty]⟩
111111

112+
theorem fg_span {s : set M} (hs : finite s) : fg (span R s) :=
113+
⟨hs.to_finset, by rw [hs.coe_to_finset]⟩
114+
115+
theorem fg_span_singleton (x : M) : fg (R ∙ x) :=
116+
fg_span (finite_singleton x)
117+
112118
theorem fg_sup {N₁ N₂ : submodule R M}
113119
(hN₁ : N₁.fg) (hN₂ : N₂.fg) : (N₁ ⊔ N₂).fg :=
114120
let ⟨t₁, ht₁⟩ := fg_def.1 hN₁, ⟨t₂, ht₂⟩ := fg_def.1 hN₂ in

0 commit comments

Comments
 (0)