Skip to content

Commit

Permalink
chore(topology): move 3 files to topology/algebra/module/ (#11242)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Jan 5, 2022
1 parent 9fd7a02 commit a1f4ac3
Show file tree
Hide file tree
Showing 16 changed files with 17 additions and 17 deletions.
2 changes: 1 addition & 1 deletion src/analysis/normed_space/banach_steinhaus.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Jireh Loreaux
-/
import analysis.normed_space.operator_norm
import topology.metric_space.baire
import topology.algebra.module
import topology.algebra.module.basic
/-!
# The Banach-Steinhaus theorem: Uniform Boundedness Principle
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/basic.lean
Expand Up @@ -7,7 +7,7 @@ import algebra.algebra.restrict_scalars
import algebra.algebra.subalgebra
import analysis.normed.group.infinite_sum
import data.matrix.basic
import topology.algebra.module
import topology.algebra.module.basic
import topology.instances.ennreal
import topology.sequences

Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/bounded_linear_maps.lean
Expand Up @@ -42,7 +42,7 @@ already expounds the theory of multilinear maps, but the `2`-variables case is s
to currently deserve its own treatment.
`is_bounded_linear_map` is effectively an unbundled version of `continuous_linear_map` (defined
in `topology.algebra.module`, theory over normed spaces developed in
in `topology.algebra.module.basic`, theory over normed spaces developed in
`analysis.normed_space.operator_norm`), albeit the name disparity. A bundled
`continuous_linear_map` is to be preferred over a `is_bounded_linear_map` hypothesis. Historical
artifact, really.
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/linear_isometry.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov, Frédéric Dupuis, Heather Macbeth
-/
import analysis.normed.group.basic
import topology.algebra.module
import topology.algebra.module.basic

/-!
# (Semi-)linear isometries
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/multilinear.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Sébastien Gouëzel
-/
import analysis.normed_space.operator_norm
import topology.algebra.multilinear
import topology.algebra.module.multilinear

/-!
# Operator norm on the space of continuous multilinear maps
Expand Down
6 changes: 3 additions & 3 deletions src/analysis/normed_space/weak_dual.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2021 Kalle Kytölä. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kalle Kytölä
-/
import topology.algebra.weak_dual_topology
import topology.algebra.module.weak_dual
import analysis.normed_space.dual
import analysis.normed_space.operator_norm

Expand Down Expand Up @@ -42,7 +42,7 @@ TODOs:
* Add that in finite dimensions, the weak-* topology and the dual norm topology coincide.
* Add that in infinite dimensions, the weak-* topology is strictly coarser than the dual norm
topology.
* Add Banach-Alaoglu theorem (general version maybe in `topology.algebra.weak_dual_topology`).
* Add Banach-Alaoglu theorem (general version maybe in `topology.algebra.module.weak_dual`).
* Add metrizability of the dual unit ball (more generally bounded subsets) of `weak_dual 𝕜 E`
under the assumption of separability of `E`. Sequential Banach-Alaoglu theorem would then follow
from the general one.
Expand All @@ -53,7 +53,7 @@ No new notation is introduced.
## Implementation notes
Weak-* topology is defined generally in the file `topology.algebra.weak_dual_topology`.
Weak-* topology is defined generally in the file `topology.algebra.module.weak_dual`.
When `E` is a normed space, the duals `dual 𝕜 E` and `weak_dual 𝕜 E` are type synonyms with
different topology instances.
Expand Down
Expand Up @@ -6,7 +6,7 @@ Authors: Kalle Kytölä
import measure_theory.measure.measure_space
import measure_theory.integral.bochner
import topology.continuous_function.bounded
import topology.algebra.weak_dual_topology
import topology.algebra.module.weak_dual

/-!
# Weak convergence of (finite) measures
Expand Down
2 changes: 1 addition & 1 deletion src/topology/algebra/algebra.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import algebra.algebra.subalgebra
import topology.algebra.module
import topology.algebra.module.basic

/-!
# Topological (sub)algebras
Expand Down
2 changes: 1 addition & 1 deletion src/topology/algebra/continuous_affine_map.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Oliver Nash
-/
import linear_algebra.affine_space.affine_map
import topology.continuous_function.basic
import topology.algebra.module
import topology.algebra.module.basic

/-!
# Continuous affine maps.
Expand Down
2 changes: 1 addition & 1 deletion src/topology/algebra/filter_basis.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Patrick Massot
-/

import order.filter.bases
import topology.algebra.module
import topology.algebra.module.basic
/-!
# Group and ring filter bases
Expand Down
File renamed without changes.
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Sébastien Gouëzel. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Sébastien Gouëzel
-/
import topology.algebra.module
import topology.algebra.module.basic
import linear_algebra.multilinear.basic

/-!
Expand Down
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2021 Kalle Kytölä. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kalle Kytölä
-/
import topology.algebra.module
import topology.algebra.module.basic

/-!
# Weak dual topology
Expand Down
2 changes: 1 addition & 1 deletion src/topology/continuous_function/algebra.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2019 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison, Nicolò Cavalleri
-/
import topology.algebra.module
import topology.algebra.module.basic
import topology.continuous_function.basic
import algebra.algebra.subalgebra
import tactic.field_simp
Expand Down
2 changes: 1 addition & 1 deletion src/topology/instances/real_vector_space.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Yury Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov
-/
import topology.algebra.module
import topology.algebra.module.basic
import topology.instances.real

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/topology/vector_bundle.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Nicolò Cavalleri, Sebastien Gouezel
-/

import topology.fiber_bundle
import topology.algebra.module
import topology.algebra.module.basic

/-!
# Topological vector bundles
Expand Down

0 comments on commit a1f4ac3

Please sign in to comment.