Documentation

Mathlib.LinearAlgebra.Projectivization.Cardinality

Cardinality of projective spaces #

We compute the cardinality of ℙ k V if k is a finite field.

ℙ k V is equivalent to the quotient of the non-zero elements of V by .

Equations
Instances For
    noncomputable def Projectivization.nonZeroEquivProjectivizationProdUnits (k : Type u_1) (V : Type u_2) [DivisionRing k] [AddCommGroup V] [Module k V] :
    { v : V // v 0 } Projectivization k V × kˣ

    The non-zero elements of V are equivalent to the product of ℙ k V with the units of k.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      If V is a finite k-module and k is finite, ℙ k V is finite.

      theorem Projectivization.card (k : Type u_1) (V : Type u_2) [DivisionRing k] [AddCommGroup V] [Module k V] :

      Fraction free cardinality formula for the points of ℙ k V if k and V are finite (for silly reasons the formula also holds when k and V are infinite). See Projectivization.card' and Projectivization.card'' for other spellings of the formula.

      theorem Projectivization.card' (k : Type u_1) (V : Type u_2) [DivisionRing k] [AddCommGroup V] [Module k V] [Finite V] :

      Cardinality formula for the points of ℙ k V if k and V are finite with less natural subtraction.

      theorem Projectivization.card'' (k : Type u_1) (V : Type u_2) [Field k] [AddCommGroup V] [Module k V] [Finite k] :

      Cardinality formula for the points of ℙ k V if k and V are finite expressed as a fraction.

      theorem Projectivization.card_of_finrank (k : Type u_1) (V : Type u_2) [Field k] [AddCommGroup V] [Module k V] [Finite k] {n : } (h : Module.finrank k V = n) :