Skip to content

Commit

Permalink
also useless
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Oct 22, 2024
1 parent 769ba16 commit 45f0066
Showing 1 changed file with 0 additions and 12 deletions.
12 changes: 0 additions & 12 deletions FltRegular/NumberTheory/Finrank.lean
Original file line number Diff line number Diff line change
Expand Up @@ -22,18 +22,6 @@ variable {R M : Type*} [CommRing R] [AddCommGroup M] [Module R M] (N : Submodule

variable [Module.Finite R M]

instance [IsDomain R] : NoZeroSMulDivisors R (M ⧸ Submodule.torsion R M) := by
constructor
intros c x hcx
rw [or_iff_not_imp_left]
intro hc
obtain ⟨x, rfl⟩ := Submodule.mkQ_surjective _ x
rw [← LinearMap.map_smul, Submodule.mkQ_apply, Submodule.Quotient.mk_eq_zero] at hcx
obtain ⟨n, hn⟩ := hcx
simp only [Submodule.mkQ_apply, Submodule.Quotient.mk_eq_zero, Submonoid.mk_smul, exists_prop]
refine ⟨n * ⟨c, mem_nonZeroDivisors_of_ne_zero hc⟩, ?_⟩
simpa [Submonoid.smul_def, smul_smul] using hn

lemma FiniteDimensional.finrank_add_finrank_quotient [IsDomain R] (N : Submodule R M) :
finrank R (M ⧸ N) + finrank R N = finrank R M := by
rw [← Cardinal.natCast_inj, Module.finrank_eq_rank, Nat.cast_add, Module.finrank_eq_rank,
Expand Down

0 comments on commit 45f0066

Please sign in to comment.