File tree Expand file tree Collapse file tree 4 files changed +547
-1
lines changed Expand file tree Collapse file tree 4 files changed +547
-1
lines changed Original file line number Diff line number Diff line change @@ -5569,6 +5569,7 @@ import Mathlib.RingTheory.OrzechProperty
55695569import Mathlib.RingTheory.Perfection
55705570import Mathlib.RingTheory.Perfectoid.Untilt
55715571import Mathlib.RingTheory.PiTensorProduct
5572+ import Mathlib.RingTheory.PicardGroup
55725573import Mathlib.RingTheory.Polynomial.Basic
55735574import Mathlib.RingTheory.Polynomial.Bernstein
55745575import Mathlib.RingTheory.Polynomial.Chebyshev
Original file line number Diff line number Diff line change @@ -5,8 +5,8 @@ Authors: Johan Commelin
55-/
66import Mathlib.LinearAlgebra.Basis.Cardinality
77import Mathlib.LinearAlgebra.DFinsupp
8- import Mathlib.LinearAlgebra.StdBasis
98import Mathlib.LinearAlgebra.Isomorphisms
9+ import Mathlib.LinearAlgebra.StdBasis
1010import Mathlib.RingTheory.Finiteness.Basic
1111
1212/-!
@@ -83,3 +83,21 @@ lemma not_finite_of_infinite_basis [Nontrivial R] {ι} [Infinite ι] (b : Basis
8383end Module
8484
8585end ModuleAndAlgebra
86+
87+ namespace Module.Finite
88+
89+ universe u
90+ variable (R : Type u) (M : Type *) [Ring R] [AddCommGroup M] [Module R M] [Module.Finite R M]
91+
92+ /-- The kernel of a random surjective linear map from a finite free module
93+ to a given finite module. -/
94+ noncomputable def kerRepr := LinearMap.ker (Finite.exists_fin' R M).choose_spec.choose
95+
96+ /-- A representative of a finite module in the same universe as the ring. -/
97+ protected abbrev repr : Type u := _ ⧸ kerRepr R M
98+
99+ /-- The representative is isomorphic to the original module. -/
100+ noncomputable def reprEquiv : Finite.repr R M ≃ₗ[R] M :=
101+ LinearMap.quotKerEquivOfSurjective _ (Finite.exists_fin' R M).choose_spec.choose_spec
102+
103+ end Module.Finite
You can’t perform that action at this time.
0 commit comments