Skip to content

Commit

Permalink
chore(order/hom): rearrange definitions of order_{hom,iso,embedding} (
Browse files Browse the repository at this point in the history
#10752)

We symmetrize the locations of `rel_{hom,iso,embedding}` and `order_{hom,iso,embedding}` by putting the `rel_` definitions in `order/rel_iso.lean` and the `order_` definitions in `order/hom/basic.lean`. (`order_hom.lean` needed to be split up to fix an import loop.) Requested by @YaelDillies.

## Moved definitions
 * `order_hom`, `order_iso`, `order_embedding` are now in `order/hom/basic.lean`
 * `order_hom.has_sup` ... `order_hom.complete_lattice` are now in `order/hom/lattice.lean`

## Other changes

Some import cleanup.
  • Loading branch information
Vierkantor committed Dec 13, 2021
1 parent b351ca9 commit 7181b3a
Show file tree
Hide file tree
Showing 16 changed files with 808 additions and 773 deletions.
4 changes: 2 additions & 2 deletions src/algebra/lie/solvable.lean
Expand Up @@ -3,9 +3,9 @@ Copyright (c) 2021 Oliver Nash. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Oliver Nash
-/
import algebra.lie.ideal_operations
import algebra.lie.abelian
import order.order_hom
import algebra.lie.ideal_operations
import order.hom.basic

/-!
# Solvable Lie algebras
Expand Down
2 changes: 1 addition & 1 deletion src/algebra/order/monoid.lean
Expand Up @@ -9,7 +9,7 @@ import algebra.group.prod
import algebra.order.monoid_lemmas
import order.bounded_order
import order.min_max
import order.rel_iso
import order.hom.basic

/-!
# Ordered monoids
Expand Down
1 change: 1 addition & 0 deletions src/combinatorics/set_family/shadow.lean
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Bhavik Mehta, Alena Gusakov, Yaël Dillies
-/
import data.finset.lattice
import logic.function.iterate

/-!
# Shadows
Expand Down
2 changes: 1 addition & 1 deletion src/data/finset/option.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov, Mario Carneiro, Sean Leather
-/
import data.finset.basic
import order.order_hom
import order.hom.basic

/-!
# Finite sets in `option α`
Expand Down
1 change: 1 addition & 0 deletions src/data/nat/fib.lean
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Kappelmann
-/
import data.nat.gcd
import logic.function.iterate
import tactic.ring

/-!
Expand Down
4 changes: 2 additions & 2 deletions src/linear_algebra/eigenspace.lean
Expand Up @@ -5,10 +5,10 @@ Authors: Alexander Bentkamp
-/

import field_theory.is_alg_closed.basic
import linear_algebra.charpoly.basic
import linear_algebra.finsupp
import linear_algebra.matrix.to_lin
import order.order_hom
import linear_algebra.charpoly.basic
import order.hom.basic

/-!
# Eigenvectors and eigenvalues
Expand Down
2 changes: 1 addition & 1 deletion src/order/category/Preorder.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Johan Commelin
-/
import category_theory.concrete_category.bundled_hom
import algebra.punit_instances
import order.order_hom
import order.hom.basic

/-! # Category of preorders -/

Expand Down
2 changes: 1 addition & 1 deletion src/order/closure.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Bhavik Mehta, Yaël Dillies
import data.set.lattice
import data.set_like.basic
import order.galois_connection
import order.order_hom
import order.hom.basic
import tactic.monotonicity

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/order/fixed_points.lean
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2017 Johannes Hölzl. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Kenny Lau, Yury Kudryashov
-/
import order.order_hom
import dynamics.fixed_points.basic
import order.hom.lattice

/-!
# Fixed point construction on complete lattices
Expand Down

0 comments on commit 7181b3a

Please sign in to comment.