File tree Expand file tree Collapse file tree 1 file changed +12
-0
lines changed Expand file tree Collapse file tree 1 file changed +12
-0
lines changed Original file line number Diff line number Diff line change @@ -42,6 +42,18 @@ theorem quotient' {R : Type*} [CommRing R] (p : ℕ) [CharP R p] (I : Ideal R)
4242 exact ⟨h x, fun h' => h'.symm ▸ I.zero_mem⟩⟩
4343#align char_p.quotient' CharP.quotient'
4444
45+ /-- `CharP.quotient'` as an `Iff`. -/
46+ theorem quotient_iff {R : Type *} [CommRing R] (n : ℕ) [CharP R n] (I : Ideal R) :
47+ CharP (R ⧸ I) n ↔ ∀ x : ℕ, ↑x ∈ I → (x : R) = 0 := by
48+ refine ⟨fun _ x hx => ?_, CharP.quotient' n I⟩
49+ rw [CharP.cast_eq_zero_iff R n, ←CharP.cast_eq_zero_iff (R ⧸ I) n _]
50+ exact (Submodule.Quotient.mk_eq_zero I).mpr hx
51+
52+ /-- `CharP.quotient_iff`, but stated in terms of inclusions of ideals. -/
53+ theorem quotient_iff_le_ker_natCast {R : Type *} [CommRing R] (n : ℕ) [CharP R n] (I : Ideal R) :
54+ CharP (R ⧸ I) n ↔ I.comap (Nat.castRingHom R) ≤ RingHom.ker (Nat.castRingHom R) := by
55+ rw [CharP.quotient_iff, RingHom.ker_eq_comap_bot]; rfl
56+
4557end CharP
4658
4759theorem Ideal.Quotient.index_eq_zero {R : Type *} [CommRing R] (I : Ideal R) :
You can’t perform that action at this time.
0 commit comments