File tree Expand file tree Collapse file tree 1 file changed +7
-0
lines changed
Mathlib/LinearAlgebra/AffineSpace Expand file tree Collapse file tree 1 file changed +7
-0
lines changed Original file line number Diff line number Diff line change @@ -113,6 +113,13 @@ instance AffineSubspace.finiteDimensional_sup (s₁ s₂ : AffineSubspace k P)
113113 rw [AffineSubspace.direction_sup hp₁ hp₂]
114114 infer_instance
115115
116+ /-- The image of a finite-dimensional affine subspace under an affine map is finite-dimensional. -/
117+ instance finiteDimensional_direction_map {V₂ P₂ : Type *} [AddCommGroup V₂] [Module k V₂]
118+ [AffineSpace V₂ P₂] (s : AffineSubspace k P) [FiniteDimensional k s.direction]
119+ (f : P →ᵃ[k] P₂) : FiniteDimensional k (s.map f).direction := by
120+ rw [map_direction]
121+ infer_instance
122+
116123/-- The `vectorSpan` of a finite subset of an affinely independent
117124family has dimension one less than its cardinality. -/
118125theorem AffineIndependent.finrank_vectorSpan_image_finset [DecidableEq P]
You can’t perform that action at this time.
0 commit comments