Skip to content

Commit

Permalink
Acl/reorg tensor product (#11282)
Browse files Browse the repository at this point in the history
Move:
* `Mathlib/Algebra/Module/DirectLimitAndTensorProduct.lean` to 
`LinearAlgebra/TensorProduct/DirectLimit.lean`
* `Mathlib/LinearAlgebra/TensorProduct` to `Mathlib/LinearAlgebra.TensorProduct.Basic.lean`
* `Mathlib/RingTheory/TensorProduct` to `Mathlib/RingTheory/TensorProduct/Basic.lean`.


This follows suggestions 1, 2, 3 of 

https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Tensor.20Products.20of.20modules.20and.20rings/near/424605543



Co-authored-by: Antoine Chambert-Loir <antoine.chambert-loir@math.univ-paris-diderot.fr>
  • Loading branch information
AntoineChambert-Loir and Antoine Chambert-Loir committed Mar 11, 2024
1 parent f8a97cf commit 0ee5f82
Show file tree
Hide file tree
Showing 32 changed files with 32 additions and 32 deletions.
8 changes: 4 additions & 4 deletions Mathlib.lean
Expand Up @@ -333,7 +333,6 @@ import Mathlib.Algebra.Module.BigOperators
import Mathlib.Algebra.Module.Bimodule
import Mathlib.Algebra.Module.CharacterModule
import Mathlib.Algebra.Module.DedekindDomain
import Mathlib.Algebra.Module.DirectLimitAndTensorProduct
import Mathlib.Algebra.Module.Equiv
import Mathlib.Algebra.Module.GradedModule
import Mathlib.Algebra.Module.Hom
Expand Down Expand Up @@ -2652,15 +2651,16 @@ import Mathlib.LinearAlgebra.TensorAlgebra.Basis
import Mathlib.LinearAlgebra.TensorAlgebra.Grading
import Mathlib.LinearAlgebra.TensorAlgebra.ToTensorPower
import Mathlib.LinearAlgebra.TensorPower
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Basic
import Mathlib.LinearAlgebra.TensorProduct.Basis
import Mathlib.LinearAlgebra.TensorProduct.DirectLimit
import Mathlib.LinearAlgebra.TensorProduct.Graded.External
import Mathlib.LinearAlgebra.TensorProduct.Graded.Internal
import Mathlib.LinearAlgebra.TensorProduct.Matrix
import Mathlib.LinearAlgebra.TensorProduct.Opposite
import Mathlib.LinearAlgebra.TensorProduct.Prod
import Mathlib.LinearAlgebra.TensorProduct.RightExactness
import Mathlib.LinearAlgebra.TensorProduct.Tower
import Mathlib.LinearAlgebra.TensorProductBasis
import Mathlib.LinearAlgebra.Trace
import Mathlib.LinearAlgebra.UnitaryGroup
import Mathlib.LinearAlgebra.Vandermonde
Expand Down Expand Up @@ -3404,7 +3404,7 @@ import Mathlib.RingTheory.Subring.Units
import Mathlib.RingTheory.Subsemiring.Basic
import Mathlib.RingTheory.Subsemiring.Order
import Mathlib.RingTheory.Subsemiring.Pointwise
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic
import Mathlib.RingTheory.Trace
import Mathlib.RingTheory.UniqueFactorizationDomain
import Mathlib.RingTheory.Valuation.Basic
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Algebra/Bilinear.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Kenny Lau, Yury Kudryashov
import Mathlib.Algebra.Algebra.Basic
import Mathlib.Algebra.Algebra.NonUnitalHom
import Mathlib.Algebra.GroupPower.IterateHom
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Basic

#align_import algebra.algebra.bilinear from "leanprover-community/mathlib"@"657df4339ae6ceada048c8a2980fb10e393143ec"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Eric Wieser
import Mathlib.CategoryTheory.Monoidal.Transport
import Mathlib.Algebra.Category.AlgebraCat.Basic
import Mathlib.Algebra.Category.ModuleCat.Monoidal.Basic
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

/-!
# The monoidal category structure on R-algebras
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jujian Zhang
-/
import Mathlib.Algebra.Category.ModuleCat.EpiMono
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

#align_import algebra.category.Module.change_of_rings from "leanprover-community/mathlib"@"56b71f0b55c03f70332b862e65c3aa1aa1249ca1"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Buzzard, Scott Morrison, Jakob von Raumer
-/
import Mathlib.Algebra.Category.ModuleCat.Basic
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Basic
import Mathlib.CategoryTheory.Monoidal.Linear

#align_import algebra.category.Module.monoidal.basic from "leanprover-community/mathlib"@"74403a3b2551b0970855e14ef5e8fd0d6af1bfc2"
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Category/Ring/Constructions.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Andrew Yang
-/
import Mathlib.CategoryTheory.Limits.Shapes.Pullbacks
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic
import Mathlib.Algebra.Category.Ring.Limits
import Mathlib.Algebra.Category.Ring.Instances
import Mathlib.CategoryTheory.Limits.Shapes.StrictInitial
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Lie/BaseChange.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Oliver Nash
import Mathlib.Algebra.Algebra.RestrictScalars
import Mathlib.Algebra.Lie.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Tower
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

#align_import algebra.lie.base_change from "leanprover-community/mathlib"@"9264b15ee696b7ca83f13c8ad67c83d6eb70b730"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Module/Bimodule.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Oliver Nash. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Oliver Nash
-/
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

#align_import algebra.module.bimodule from "leanprover-community/mathlib"@"58cef51f7a819e7227224461e392dee423302f2d"

Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Data/Matrix/Kronecker.lean
Expand Up @@ -7,8 +7,8 @@ import Mathlib.Data.Matrix.Basic
import Mathlib.Data.Matrix.Block
import Mathlib.LinearAlgebra.Matrix.Determinant
import Mathlib.LinearAlgebra.Matrix.NonsingularInverse
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.RingTheory.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Basic
import Mathlib.RingTheory.TensorProduct.Basic

#align_import data.matrix.kronecker from "leanprover-community/mathlib"@"3e068ece210655b7b9a9477c3aff38a492400aa1"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/FieldTheory/Adjoin.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Thomas Browning, Patrick Lutz
import Mathlib.FieldTheory.IntermediateField
import Mathlib.FieldTheory.Separable
import Mathlib.FieldTheory.SplittingField.IsSplittingField
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

#align_import field_theory.adjoin from "leanprover-community/mathlib"@"df76f43357840485b9d04ed5dee5ab115d420e87"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/CliffordAlgebra/BaseChange.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Eric Wieser
import Mathlib.LinearAlgebra.QuadraticForm.TensorProduct
import Mathlib.LinearAlgebra.CliffordAlgebra.Conjugation
import Mathlib.LinearAlgebra.TensorProduct.Opposite
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

/-!
# The base change of a clifford algebra
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/DirectSum/TensorProduct.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2018 Kenny Lau. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kenny Lau, Mario Carneiro, Eric Wieser
-/
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Basic
import Mathlib.Algebra.DirectSum.Module

#align_import linear_algebra.direct_sum.tensor_product from "leanprover-community/mathlib"@"9b9d125b7be0930f564a68f1d73ace10cf46064d"
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/Dual.lean
Expand Up @@ -9,7 +9,7 @@ import Mathlib.LinearAlgebra.FreeModule.Finite.Basic
import Mathlib.LinearAlgebra.FreeModule.StrongRankCondition
import Mathlib.LinearAlgebra.Projection
import Mathlib.LinearAlgebra.SesquilinearForm
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

#align_import linear_algebra.dual from "leanprover-community/mathlib"@"b1c017582e9f18d8494e5c18602a8cb4a6f843ac"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/FreeModule/Basic.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Riccardo Brasca
-/
import Mathlib.Data.Finsupp.Fintype
import Mathlib.LinearAlgebra.TensorProductBasis
import Mathlib.LinearAlgebra.TensorProduct.Basis

#align_import linear_algebra.free_module.basic from "leanprover-community/mathlib"@"4e7e7009099d4a88a750de710909b95487bf0124"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Eric Wieser
-/
import Mathlib.LinearAlgebra.Multilinear.Basic
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Basic

#align_import linear_algebra.multilinear.tensor_product from "leanprover-community/mathlib"@"ce11c3c2a285bbe6937e26d9792fda4e51f3fe1a"

Expand Down
File renamed without changes.
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Eric Wieser
-/
import Mathlib.Data.Int.Order.Units
import Mathlib.Data.ZMod.IntUnitsPower
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic
import Mathlib.LinearAlgebra.DirectSum.TensorProduct
import Mathlib.Algebra.DirectSum.Algebra

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/TensorProduct/Matrix.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Eric Wieser
-/
import Mathlib.Data.Matrix.Kronecker
import Mathlib.LinearAlgebra.Matrix.ToLin
import Mathlib.LinearAlgebra.TensorProductBasis
import Mathlib.LinearAlgebra.TensorProduct.Basis

#align_import linear_algebra.tensor_product.matrix from "leanprover-community/mathlib"@"f784cc6142443d9ee623a20788c282112c322081"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/TensorProduct/Opposite.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2023 Eric Wieser. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Eric Wieser
-/
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic
import Mathlib.Algebra.Algebra.Opposite

/-! # `MulOpposite` distributes over `⊗`
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/TensorProduct/Prod.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2023 Eric Wieser. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Eric Wieser
-/
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Basic
import Mathlib.LinearAlgebra.Prod

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/TensorProduct/RightExactness.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Antoine Chambetr-Loir
-/

import Mathlib.Algebra.Exact
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

/-! # Right-exactness properties of tensor product
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/TensorProduct/Tower.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Scott Morrison, Johan Commelin, Eric Wieser
-/
import Mathlib.Algebra.Algebra.Tower
import Mathlib.LinearAlgebra.Basic
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Basic

#align_import ring_theory.tensor_product from "leanprover-community/mathlib"@"88fcdc3da43943f5b01925deddaa5bf0c0e85e4e"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RepresentationTheory/Basic.lean
Expand Up @@ -9,7 +9,7 @@ import Mathlib.Algebra.Module.LinearMap.Basic
import Mathlib.Algebra.MonoidAlgebra.Basic
import Mathlib.LinearAlgebra.Dual
import Mathlib.LinearAlgebra.Contraction
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

#align_import representation_theory.basic from "leanprover-community/mathlib"@"c04bc6e93e23aa0182aba53661a2211e80b6feac"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Bialgebra.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Ali Ramsey, Kevin Buzzard
-/
import Mathlib.RingTheory.Coalgebra
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

/-!
# Bialgebras
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Coalgebra.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Ali Ramsey, Eric Wieser
-/
import Mathlib.LinearAlgebra.Finsupp
import Mathlib.LinearAlgebra.Prod
import Mathlib.LinearAlgebra.TensorProduct
import Mathlib.LinearAlgebra.TensorProduct.Basic

/-!
# Coalgebras
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/IntegralClosure.lean
Expand Up @@ -10,7 +10,7 @@ import Mathlib.RingTheory.Adjoin.FG
import Mathlib.RingTheory.FiniteType
import Mathlib.RingTheory.Polynomial.ScaleRoots
import Mathlib.RingTheory.Polynomial.Tower
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

#align_import ring_theory.integral_closure from "leanprover-community/mathlib"@"641b6a82006416ec431b2987b354af9311fed4f2"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/IsTensorProduct.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Andrew Yang. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Andrew Yang
-/
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic
import Mathlib.Algebra.Module.ULift

#align_import ring_theory.is_tensor_product from "leanprover-community/mathlib"@"c4926d76bb9c5a4a62ed2f03d998081786132105"
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/MatrixAlgebra.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison, Eric Wieser
-/
import Mathlib.Data.Matrix.Basis
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

#align_import ring_theory.matrix_algebra from "leanprover-community/mathlib"@"6c351a8fb9b06e5a542fdf427bfb9f46724f9453"

Expand Down
File renamed without changes.
2 changes: 1 addition & 1 deletion test/instance_diamonds.lean
Expand Up @@ -10,7 +10,7 @@ import Mathlib.GroupTheory.GroupAction.Units
import Mathlib.Data.Complex.Module
import Mathlib.RingTheory.Algebraic
import Mathlib.Data.ZMod.Basic
import Mathlib.RingTheory.TensorProduct
import Mathlib.RingTheory.TensorProduct.Basic

/-! # Tests that instances do not form diamonds -/

Expand Down

0 comments on commit 0ee5f82

Please sign in to comment.