Documentation

Mathlib.Topology.Algebra.Module.Determinant

The determinant of a continuous linear map. #

@[reducible]
noncomputable def ContinuousLinearMap.det {R : Type u_1} [CommRing R] {M : Type u_2} [TopologicalSpace M] [AddCommGroup M] [Module R M] (A : M →L[R] M) :
R

The determinant of a continuous linear map, mainly as a convenience device to be able to write A.det instead of (A : M →ₗ[R] M).det.

Equations
Instances For