Skip to content

Commit

Permalink
chore(order/bounded_order): remove unnecessary imports (#17180)
Browse files Browse the repository at this point in the history


Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Oct 27, 2022
1 parent 6bc0c19 commit c571859
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 1 deletion.
2 changes: 1 addition & 1 deletion src/order/bounded_order.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl
-/
import order.lattice
import logic.equiv.basic
import data.option.basic

/-!
# ⊤ and ⊥, bounded lattices and variants
Expand Down
1 change: 1 addition & 0 deletions src/order/symm_diff.lean
Expand Up @@ -5,6 +5,7 @@ Authors: Adam Topaz, Bryan Gin-ge Chen, Yaël Dillies
-/

import order.boolean_algebra
import logic.equiv.basic

/-!
# Symmetric difference and bi-implication
Expand Down

0 comments on commit c571859

Please sign in to comment.