Skip to content

Commit 9127890

Browse files
committed
chore(LinearAlgebra/Span): split off definition of Submodule.span (#18618)
This PR creates a new file `LinearAlgebra.Span.Defs` which contains the definition of a submodule span and some elementary results. Everything that needs heavier imports gets moved to `LinearAlgebra.Span.Basic`.
1 parent 2c03193 commit 9127890

File tree

15 files changed

+551
-500
lines changed

15 files changed

+551
-500
lines changed

Mathlib.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3369,7 +3369,8 @@ import Mathlib.LinearAlgebra.RootSystem.RootPositive
33693369
import Mathlib.LinearAlgebra.SModEq
33703370
import Mathlib.LinearAlgebra.Semisimple
33713371
import Mathlib.LinearAlgebra.SesquilinearForm
3372-
import Mathlib.LinearAlgebra.Span
3372+
import Mathlib.LinearAlgebra.Span.Basic
3373+
import Mathlib.LinearAlgebra.Span.Defs
33733374
import Mathlib.LinearAlgebra.StdBasis
33743375
import Mathlib.LinearAlgebra.SymplecticGroup
33753376
import Mathlib.LinearAlgebra.TensorAlgebra.Basic

Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Jireh Loreaux
55
-/
66
import Mathlib.Algebra.Algebra.NonUnitalHom
77
import Mathlib.Data.Set.UnionLift
8-
import Mathlib.LinearAlgebra.Span
8+
import Mathlib.LinearAlgebra.Span.Basic
99
import Mathlib.RingTheory.NonUnitalSubring.Basic
1010

1111
/-!

Mathlib/Algebra/Algebra/Tower.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Kenny Lau, Anne Baanen
55
-/
66
import Mathlib.Algebra.Algebra.Equiv
7-
import Mathlib.LinearAlgebra.Span
7+
import Mathlib.LinearAlgebra.Span.Basic
88

99
/-!
1010
# Towers of algebras

Mathlib/Algebra/Category/ModuleCat/Tannaka.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Kim Morrison
55
-/
66
import Mathlib.Algebra.Category.ModuleCat.Basic
7-
import Mathlib.LinearAlgebra.Span
7+
import Mathlib.LinearAlgebra.Span.Basic
88

99
/-!
1010
# Tannaka duality for rings

Mathlib/Algebra/Module/Submodule/Bilinear.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2019 Kenny Lau. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Kenny Lau, Eric Wieser
55
-/
6-
import Mathlib.LinearAlgebra.Span
6+
import Mathlib.LinearAlgebra.Span.Basic
77
import Mathlib.LinearAlgebra.BilinearMap
88

99
/-!

Mathlib/LinearAlgebra/Basis/Defs.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Johannes Hölzl, Mario Carneiro, Alexander Bentkamp
55
-/
66
import Mathlib.LinearAlgebra.Finsupp.LinearCombination
7-
import Mathlib.LinearAlgebra.Span
7+
import Mathlib.LinearAlgebra.Span.Basic
88

99
/-!
1010
# Bases

Mathlib/LinearAlgebra/FiniteSpan.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Oliver Nash, Deepro Choudhury
55
-/
66
import Mathlib.GroupTheory.OrderOfElement
7-
import Mathlib.LinearAlgebra.Span
7+
import Mathlib.LinearAlgebra.Span.Defs
88
import Mathlib.Algebra.Module.Equiv.Basic
99

1010
/-!

Mathlib/LinearAlgebra/Finsupp/Span.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Johannes Hölzl
55
-/
66
import Mathlib.LinearAlgebra.Finsupp.Defs
7-
import Mathlib.LinearAlgebra.Span
7+
import Mathlib.LinearAlgebra.Span.Basic
88

99
/-!
1010
# Finitely supported functions and spans

Mathlib/LinearAlgebra/Finsupp/Supported.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Johannes Hölzl
55
-/
66
import Mathlib.Algebra.Module.Submodule.Range
77
import Mathlib.LinearAlgebra.Finsupp.LSum
8-
import Mathlib.LinearAlgebra.Span
8+
import Mathlib.LinearAlgebra.Span.Defs
99

1010
/-!
1111
# `Finsupp`s supported on a given submodule

Mathlib/LinearAlgebra/Prod.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Johannes Hölzl, Mario Carneiro, Kevin Buzzard, Yury Kudryashov, Eric Wieser
55
-/
66
import Mathlib.Algebra.Algebra.Prod
7-
import Mathlib.LinearAlgebra.Span
7+
import Mathlib.LinearAlgebra.Span.Basic
88
import Mathlib.Order.PartialSups
99

1010
/-! ### Products of modules

0 commit comments

Comments
 (0)