Skip to content

Commit

Permalink
refactor(analysis/convex/cone): move cone.lean to cone/basic.lean (#1…
Browse files Browse the repository at this point in the history
…6270)

Part of #16266 

I intend to create another file for `proper_cone`, which for cyclic import reasons cannot be included in cone.lean.
So I want to move cone.lean to cone/basic.lean and create cone/proper.lean in a separate PR.
  • Loading branch information
apurvnakade committed Aug 31, 2022
1 parent 2d30ffc commit d44692a
Show file tree
Hide file tree
Showing 3 changed files with 2 additions and 3 deletions.
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2020 Yury Kudryashov All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov, Frédéric Dupuis
-/
import analysis.convex.hull
import analysis.inner_product_space.projection

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/hahn_banach/extension.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, Heather Macbeth
-/
import analysis.convex.cone
import analysis.convex.cone.basic
import analysis.normed_space.is_R_or_C
import analysis.normed_space.extend

Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/hahn_banach/separation.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Bhavik Mehta All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Bhavik Mehta, Yaël Dillies
-/
import analysis.convex.cone
import analysis.convex.cone.basic
import analysis.convex.gauge

/-!
Expand Down

0 comments on commit d44692a

Please sign in to comment.