Projective Spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file contains the definition of the projectivization of a vector space over a field, as well as the bijection between said projectivization and the collection of all one dimensional subspaces of the vector space.
Notation #
ℙ K V
is notation for projectivization K V
, the projectivization of a K
-vector space V
.
Constructing terms of ℙ K V
. #
We have three ways to construct terms of ℙ K V
:
projectivization.mk K v hv
wherev : V
andhv : v ≠ 0
.projectivization.mk' K v
wherev : { w : V // w ≠ 0 }
.projectivization.mk'' H h
whereH : submodule K V
andh : finrank H = 1
.
Other definitions #
- For
v : ℙ K V
,v.submodule
gives the corresponding submodule ofV
. projectivization.equiv_submodule
is the equivalence betweenℙ K V
and{ H : submodule K V // finrank H = 1 }
.- For
v : ℙ K V
,v.rep : V
is a representative ofv
.
The setoid whose quotient is the projectivization of V
.
Equations
The projectivization of the K
-vector space V
.
The notation ℙ K V
is preferred.
Equations
- ℙ K V = quotient (projectivization_setoid K V)
Instances for projectivization
Construct an element of the projectivization from a nonzero vector.
Equations
- projectivization.mk K v hv = quotient.mk' ⟨v, hv⟩
A variant of projectivization.mk
in terms of a subtype. mk
is preferred.
Equations
Choose a representative of v : projectivization K V
in V
.
Equations
- v.rep = ↑(quotient.out' v)
Consider an element of the projectivization as a submodule of V
.
Equations
- v.submodule = quotient.lift_on' v (λ (v : {v // v ≠ 0}), submodule.span K {↑v}) projectivization.submodule._proof_1
Instances for ↥projectivization.submodule
Two nonzero vectors go to the same point in projective space if and only if one is a scalar multiple of the other.
An induction principle for projectivization
.
Use as induction v using projectivization.ind
.
The equivalence between the projectivization and the collection of subspaces of dimension 1.
Equations
- projectivization.equiv_submodule K V = equiv.of_bijective (λ (v : ℙ K V), ⟨v.submodule, _⟩) _
Construct an element of the projectivization from a subspace of dimension 1.
Equations
- projectivization.mk'' H h = ⇑((projectivization.equiv_submodule K V).symm) ⟨H, h⟩
An injective semilinear map of vector spaces induces a map on projective spaces.
Equations
- projectivization.map f hf = quotient.map' (λ (v : {v // v ≠ 0}), ⟨⇑f ↑v, _⟩) _
Mapping with respect to a semilinear map over an isomorphism of fields yields an injective map on projective spaces.