We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 36a2b22 commit f9aa536Copy full SHA for f9aa536
Mathlib/RingTheory/PrincipalIdealDomain.lean
@@ -560,3 +560,12 @@ theorem nonPrincipals_zorn (c : Set (Ideal R)) (hs : c ⊆ { I : Ideal R | ¬I.I
560
exact hs ⟨⟨x, rfl⟩⟩
561
562
end PrincipalOfPrime_old
563
+
564
+open Ideal in
565
+lemma span_singleton_inf_span_singleton [EuclideanDomain R] [GCDMonoid R] (n m : R) :
566
+ span {n} ⊓ span {m} = span {lcm n m} := by
567
+ rw [Ideal.ext_iff]
568
+ intro x
569
+ rw [Ideal.mem_inf]
570
+ simp only [Ideal.mem_span_singleton]
571
+ exact lcm_dvd_iff.symm
0 commit comments