Skip to content

Commit

Permalink
chore(*): minor import cleanup (#3546)
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 Jul 25, 2020
1 parent 2a456a9 commit 0379d3a
Show file tree
Hide file tree
Showing 8 changed files with 7 additions and 11 deletions.
3 changes: 2 additions & 1 deletion src/algebra/group/pi.lean
Expand Up @@ -3,7 +3,8 @@ Copyright (c) 2018 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Simon Hudon, Patrick Massot
-/
import algebra.ordered_group tactic.pi_instances
import algebra.ordered_group
import tactic.pi_instances
/-!
# Pi instances for groups and monoids
Expand Down
4 changes: 3 additions & 1 deletion src/algebra/ring/pi.lean
Expand Up @@ -3,7 +3,9 @@ Copyright (c) 2018 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Simon Hudon, Patrick Massot
-/
import tactic.pi_instances algebra.group.pi algebra.ring.basic
import tactic.pi_instances
import algebra.group.pi
import algebra.ring.basic

/-!
# Pi instances for ring
Expand Down
1 change: 0 additions & 1 deletion src/category_theory/endomorphism.lean
Expand Up @@ -5,7 +5,6 @@ Authors: Yury Kudryashov, Scott Morrison, Simon Hudon
Definition and basic properties of endomorphisms and automorphisms of an object in a category.
-/
import category_theory.category
import category_theory.groupoid
import data.equiv.mul_add

Expand Down
1 change: 0 additions & 1 deletion src/category_theory/groupoid.lean
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2018 Reid Barton All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Reid Barton, Scott Morrison, David Wärn
-/
import category_theory.category
import category_theory.epi_mono

namespace category_theory
Expand Down
2 changes: 1 addition & 1 deletion src/data/equiv/encodable/lattice.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Author: Floris van Doorn
-/
import data.equiv.encodable.basic
import data.finset
import data.finset.basic
import data.set.disjointed
/-!
# Lattice operations on encodable types
Expand Down
3 changes: 1 addition & 2 deletions src/data/indicator_function.lean
Expand Up @@ -4,8 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Zhouhang Zhou
-/
import algebra.group.pi
import algebra.module.basic
import data.set.disjointed
import group_theory.group_action
import data.support
import data.finset.lattice

Expand Down
1 change: 0 additions & 1 deletion src/data/real/nnreal.lean
Expand Up @@ -7,7 +7,6 @@ Nonnegative real numbers.
-/
import algebra.linear_ordered_comm_group_with_zero
import algebra.big_operators.ring
import data.finset.lattice
import data.real.basic
import data.indicator_function

Expand Down
3 changes: 0 additions & 3 deletions src/topology/algebra/monoid.lean
Expand Up @@ -5,11 +5,8 @@ Authors: Johannes Hölzl, Mario Carneiro
Theory of topological monoids.
-/

import topology.continuous_on
import algebra.group.pi
import group_theory.submonoid.basic
import algebra.group.prod
import deprecated.submonoid

open classical set filter topological_space
Expand Down

0 comments on commit 0379d3a

Please sign in to comment.