Documentation

Mathlib.LinearAlgebra.Projectivization.Subspace

Subspaces of Projective Space #

In this file we define subspaces of a projective space, and show that the subspaces of a projective space form a complete lattice under inclusion.

Implementation Details #

A subspace of a projective space ℙ K V is defined to be a structure consisting of a subset of ℙ K V such that if two nonzero vectors in V determine points in ℙ K V which are in the subset, and the sum of the two vectors is nonzero, then the point determined by the sum of the two vectors is also in the subset.

Results #

Future Work #

structure Projectivization.Subspace (K : Type u_1) (V : Type u_2) [Field K] [AddCommGroup V] [Module K V] :
Type u_2

A subspace of a projective space is a structure consisting of a set of points such that: If two nonzero vectors determine points which are in the set, and the sum of the two vectors is nonzero, then the point determined by the sum is also in the set.

Instances For
    theorem Projectivization.Subspace.ext {K : Type u_1} {V : Type u_2} {inst✝ : Field K} {inst✝¹ : AddCommGroup V} {inst✝² : Module K V} {x y : Subspace K V} (carrier : x.carrier = y.carrier) :
    x = y
    @[simp]
    theorem Projectivization.Subspace.mem_carrier_iff {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] (A : Subspace K V) (x : Projectivization K V) :
    x A.carrier x A
    theorem Projectivization.Subspace.mem_add {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] (T : Subspace K V) (v w : V) (hv : v 0) (hw : w 0) (hvw : v + w 0) :
    Projectivization.mk K v hv TProjectivization.mk K w hw TProjectivization.mk K (v + w) hvw T
    inductive Projectivization.Subspace.spanCarrier {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] (S : Set (Projectivization K V)) :

    The span of a set of points in a projective space is defined inductively to be the set of points which contains the original set, and contains all points determined by the (nonzero) sum of two nonzero vectors, each of which determine points in the span.

    Instances For
      def Projectivization.Subspace.span {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] (S : Set (Projectivization K V)) :

      The span of a set of points in projective space is a subspace.

      Equations
      Instances For
        theorem Projectivization.Subspace.subset_span {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] (S : Set (Projectivization K V)) :
        S (span S)

        The span of a set of points contains the set of points.

        The span of a set of points is a Galois insertion between sets of points of a projective space and subspaces of the projective space.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem Projectivization.Subspace.span_coe {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] (W : Subspace K V) :
          span W = W

          The span of a subspace is the subspace.

          instance Projectivization.Subspace.instInf {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] :

          The infimum of two subspaces exists.

          Equations
          instance Projectivization.Subspace.instInfSet {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] :

          Infimums of arbitrary collections of subspaces exist.

          Equations

          The subspaces of a projective space form a complete lattice.

          Equations
          @[simp]
          theorem Projectivization.Subspace.span_empty {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] :

          The span of the empty set is the bottom of the lattice of subspaces.

          @[simp]

          The span of the entire projective space is the top of the lattice of subspaces.

          theorem Projectivization.Subspace.span_le_subspace_iff {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {S : Set (Projectivization K V)} {W : Subspace K V} :
          span S W S W

          The span of a set of points is contained in a subspace if and only if the set of points is contained in the subspace.

          If a set of points is a subset of another set of points, then its span will be contained in the span of that set.

          theorem Projectivization.Subspace.span_le_span {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {s t : Set (Projectivization K V)} (hst : s t) :
          theorem Projectivization.Subspace.subset_span_trans {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {S T U : Set (Projectivization K V)} (hST : S (span T)) (hTU : T (span U)) :
          S (span U)
          theorem Projectivization.Subspace.span_union {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] (S T : Set (Projectivization K V)) :
          span (S T) = span S span T

          The supremum of two subspaces is equal to the span of their union.

          theorem Projectivization.Subspace.span_iUnion {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {ι : Sort u_3} (s : ιSet (Projectivization K V)) :
          span (⋃ (i : ι), s i) = ⨆ (i : ι), span (s i)

          The supremum of a collection of subspaces is equal to the span of the union of the collection.

          theorem Projectivization.Subspace.sup_span {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {S : Set (Projectivization K V)} {W : Subspace K V} :
          W span S = span (W S)

          The supremum of a subspace and the span of a set of points is equal to the span of the union of the subspace and the set of points.

          theorem Projectivization.Subspace.span_sup {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {S : Set (Projectivization K V)} {W : Subspace K V} :
          span S W = span (S W)
          theorem Projectivization.Subspace.mem_span {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {S : Set (Projectivization K V)} (u : Projectivization K V) :
          u span S ∀ (W : Subspace K V), S Wu W

          A point in a projective space is contained in the span of a set of points if and only if the point is contained in all subspaces of the projective space which contain the set of points.

          theorem Projectivization.Subspace.span_eq_sInf {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {S : Set (Projectivization K V)} :
          span S = sInf {W : Subspace K V | S W}

          The span of a set of points in a projective space is equal to the infimum of the collection of subspaces which contain the set.

          theorem Projectivization.Subspace.span_eq_of_le {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {S : Set (Projectivization K V)} {W : Subspace K V} (hS : S W) (hW : W span S) :
          span S = W

          If a set of points in projective space is contained in a subspace, and that subspace is contained in the span of the set of points, then the span of the set of points is equal to the subspace.

          theorem Projectivization.Subspace.span_eq_span_iff {K : Type u_1} {V : Type u_2} [Field K] [AddCommGroup V] [Module K V] {S T : Set (Projectivization K V)} :
          span S = span T S (span T) T (span S)

          The spans of two sets of points in a projective space are equal if and only if each set of points is contained in the span of the other set.