Documentation

Mathlib.LinearAlgebra.Projectivization.Independence

Independence in Projective Space #

In this file we define independence and dependence of families of elements in projective space.

Implementation Details #

We use an inductive definition to define the independence of points in projective space, where the only constructor assumes an independent family of vectors from the ambient vector space. Similarly for the definition of dependence.

Results #

Future Work #

inductive Projectivization.Independent {ι : Type u_1} {K : Type u_2} {V : Type u_3} [DivisionRing K] [AddCommGroup V] [Module K V] :
(ιProjectivization K V)Prop

A linearly independent family of nonzero vectors gives an independent family of points in projective space.

Instances For
    theorem Projectivization.independent_iff {ι : Type u_1} {K : Type u_2} {V : Type u_3} [DivisionRing K] [AddCommGroup V] [Module K V] {f : ιProjectivization K V} :

    A family of points in a projective space is independent if and only if the representative vectors determined by the family are linearly independent.

    A family of points in projective space is independent if and only if the family of submodules which the points determine is independent in the lattice-theoretic sense.

    inductive Projectivization.Dependent {ι : Type u_1} {K : Type u_2} {V : Type u_3} [DivisionRing K] [AddCommGroup V] [Module K V] :
    (ιProjectivization K V)Prop

    A linearly dependent family of nonzero vectors gives a dependent family of points in projective space.

    Instances For
      theorem Projectivization.dependent_iff {ι : Type u_1} {K : Type u_2} {V : Type u_3} [DivisionRing K] [AddCommGroup V] [Module K V] {f : ιProjectivization K V} :

      A family of points in a projective space is dependent if and only if their representatives are linearly dependent.

      Dependence is the negation of independence.

      Independence is the negation of dependence.

      @[simp]

      Two points in a projective space are dependent if and only if they are equal.

      @[simp]

      Two points in a projective space are independent if and only if the points are not equal.