Skip to content

Commit

Permalink
move(order/hom/order): Move from order.hom.lattice (#11601)
Browse files Browse the repository at this point in the history
Rename `order.hom.lattice` into `order.hom.order` to make space for lattice homomorphisms, as opposed to the lattice of order homomorphisms.
  • Loading branch information
YaelDillies committed Jan 22, 2022
1 parent 206b56e commit bd3b892
Show file tree
Hide file tree
Showing 3 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion src/order/fixed_points.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Kenny Lau, Yury Kudryashov
-/
import dynamics.fixed_points.basic
import order.hom.lattice
import order.hom.order

/-!
# Fixed point construction on complete lattices
Expand Down
File renamed without changes.
2 changes: 1 addition & 1 deletion src/order/omega_complete_partial_order.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Simon Hudon
-/
import control.monad.basic
import data.part
import order.hom.lattice
import order.hom.order
import tactic.monotonicity
import tactic.wlog

Expand Down

0 comments on commit bd3b892

Please sign in to comment.