Skip to content

Commit

Permalink
move(analysis/normed/order/basic): Move from `analysis.normed_space.o…
Browse files Browse the repository at this point in the history
…rdered` (#17239)

Rename `analysis.normed_space.ordered` to `analysis.normed.order.basic` because:
* It wasn't mentioning `normed_space` at all
* I am about to add properties of upper/lower sets in normed ordered groups
  • Loading branch information
YaelDillies committed Oct 29, 2022
1 parent 62c0a4e commit 76ec0e5
Show file tree
Hide file tree
Showing 7 changed files with 6 additions and 6 deletions.
2 changes: 1 addition & 1 deletion src/analysis/asymptotics/asymptotic_equivalent.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Anatole Dedecker
-/
import analysis.asymptotics.asymptotics
import analysis.normed_space.ordered
import analysis.normed.order.basic

/-!
# Asymptotic equivalence
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/asymptotics/specific_asymptotics.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2021 Anatole Dedecker. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Anatole Dedecker
-/
import analysis.normed_space.ordered
import analysis.normed.order.basic
import analysis.asymptotics.asymptotics

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/asymptotics/superpolynomial_decay.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Devon Tuma
-/
import analysis.asymptotics.asymptotics
import analysis.normed_space.ordered
import analysis.normed.order.basic
import data.polynomial.eval
import topology.algebra.order.liminf_limsup

Expand Down
2 changes: 1 addition & 1 deletion src/analysis/convex/exposed.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Yaël Dillies, Bhavik Mehta
-/
import analysis.convex.extreme
import analysis.convex.function
import analysis.normed_space.ordered
import analysis.normed.order.basic

/-!
# Exposed sets
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/convex/strict_convex_space.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Yaël Dillies, Yury Kudryashov
-/
import analysis.convex.strict
import analysis.convex.topology
import analysis.normed_space.ordered
import analysis.normed.order.basic
import analysis.normed_space.pointwise
import analysis.normed_space.affine_isometry

Expand Down
2 changes: 1 addition & 1 deletion src/analysis/locally_convex/basic.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Jean Lo, Bhavik Mehta, Yaël Dillies
import analysis.convex.basic
import analysis.convex.hull
import analysis.normed_space.lattice_ordered_group
import analysis.normed_space.ordered
import analysis.normed.order.basic

/-!
# Local convexity
Expand Down
File renamed without changes.

0 comments on commit 76ec0e5

Please sign in to comment.