Skip to content

Commit 45f0066

Browse files
also useless
1 parent 769ba16 commit 45f0066

File tree

1 file changed

+0
-12
lines changed

1 file changed

+0
-12
lines changed

FltRegular/NumberTheory/Finrank.lean

-12
Original file line numberDiff line numberDiff line change
@@ -22,18 +22,6 @@ variable {R M : Type*} [CommRing R] [AddCommGroup M] [Module R M] (N : Submodule
2222

2323
variable [Module.Finite R M]
2424

25-
instance [IsDomain R] : NoZeroSMulDivisors R (M ⧸ Submodule.torsion R M) := by
26-
constructor
27-
intros c x hcx
28-
rw [or_iff_not_imp_left]
29-
intro hc
30-
obtain ⟨x, rfl⟩ := Submodule.mkQ_surjective _ x
31-
rw [← LinearMap.map_smul, Submodule.mkQ_apply, Submodule.Quotient.mk_eq_zero] at hcx
32-
obtain ⟨n, hn⟩ := hcx
33-
simp only [Submodule.mkQ_apply, Submodule.Quotient.mk_eq_zero, Submonoid.mk_smul, exists_prop]
34-
refine ⟨n * ⟨c, mem_nonZeroDivisors_of_ne_zero hc⟩, ?_⟩
35-
simpa [Submonoid.smul_def, smul_smul] using hn
36-
3725
lemma FiniteDimensional.finrank_add_finrank_quotient [IsDomain R] (N : Submodule R M) :
3826
finrank R (M ⧸ N) + finrank R N = finrank R M := by
3927
rw [← Cardinal.natCast_inj, Module.finrank_eq_rank, Nat.cast_add, Module.finrank_eq_rank,

0 commit comments

Comments
 (0)