Skip to content

Commit

Permalink
refactor(linear_algebra/basic): split file (#12637)
Browse files Browse the repository at this point in the history
`linear_algebra.basic` has become a 2800 line monster, with lots of imports.

This is some further work on splitting it into smaller pieces, by extracting everything about (or needing) `span` to `linear_algebra.span`.



Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Mar 15, 2022
1 parent 2ad9b39 commit 585d641
Show file tree
Hide file tree
Showing 11 changed files with 842 additions and 765 deletions.
2 changes: 1 addition & 1 deletion src/algebra/algebra/basic.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kenny Lau, Yury Kudryashov
-/
import algebra.module.basic
import linear_algebra.basic
import linear_algebra.span
import tactic.abel
import data.equiv.ring_aut

Expand Down
2 changes: 1 addition & 1 deletion src/algebra/module/submodule_pointwise.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Eric Wieser
-/
import group_theory.subgroup.pointwise
import linear_algebra.basic
import linear_algebra.span

/-! # Pointwise instances on `submodule`s
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/finite_dimension.lean
Expand Up @@ -684,7 +684,7 @@ let ⟨g, hg⟩ := (f : E →ₗ[𝕜] F).exists_right_inverse_of_surjective hf
⟨g.to_continuous_linear_map, continuous_linear_map.ext $ linear_map.ext_iff.1 hg⟩

lemma closed_embedding_smul_left {c : E} (hc : c ≠ 0) : closed_embedding (λ x : 𝕜, x • c) :=
linear_equiv.closed_embedding_of_injective (linear_equiv.ker_to_span_singleton 𝕜 E hc)
linear_equiv.closed_embedding_of_injective (linear_map.ker_to_span_singleton 𝕜 E hc)

/- `smul` is a closed map in the first argument. -/
lemma is_closed_map_smul_left (c : E) : is_closed_map (λ x : 𝕜, x • c) :=
Expand Down

0 comments on commit 585d641

Please sign in to comment.