Skip to content

Commit

Permalink
chore(*): remove unnecessary import tactic (#7560)
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 May 10, 2021
1 parent 17cba54 commit ac1f3df
Show file tree
Hide file tree
Showing 9 changed files with 6 additions and 8 deletions.
1 change: 1 addition & 0 deletions archive/100-theorems-list/83_friendship_graphs.lean
Expand Up @@ -8,6 +8,7 @@ import linear_algebra.char_poly.coeff
import data.int.modeq
import data.zmod.basic
import tactic.interval_cases
import tactic.omega

/-!
# The Friendship Theorem
Expand Down
1 change: 0 additions & 1 deletion src/category_theory/limits/kan_extension.lean
Expand Up @@ -7,7 +7,6 @@ import category_theory.punit
import category_theory.structured_arrow
import category_theory.limits.functor_category
import category_theory.limits.shapes.terminal
import tactic

/-!
Expand Down
1 change: 0 additions & 1 deletion src/combinatorics/colex.lean
Expand Up @@ -6,7 +6,6 @@ Authors: Bhavik Mehta, Alena Gusakov
import data.finset
import data.fintype.basic
import algebra.geom_sum
import tactic

/-!
# Colex
Expand Down
3 changes: 2 additions & 1 deletion src/data/nat/fib.lean
Expand Up @@ -4,8 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Kappelmann
-/
import data.stream.basic
import tactic
import data.nat.gcd
import tactic.ring

/-!
# The Fibonacci Sequence
Expand Down
2 changes: 0 additions & 2 deletions src/data/set/constructions.lean
Expand Up @@ -3,8 +3,6 @@ Copyright (c) 2020 Adam Topaz. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Adam Topaz
-/

import tactic
import data.finset.basic

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/number_theory/arithmetic_function.lean
Expand Up @@ -7,7 +7,7 @@ import algebra.big_operators.ring
import number_theory.divisors
import algebra.squarefree
import algebra.invertible

import tactic.omega
/-!
# Arithmetic Functions and Dirichlet Convolution
Expand Down
2 changes: 1 addition & 1 deletion src/number_theory/divisors.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Aaron Anderson
-/
import algebra.big_operators.order
import tactic
import data.finset.intervals
import data.nat.prime

/-!
Expand Down
1 change: 0 additions & 1 deletion src/ring_theory/polynomial/symmetric.lean
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2020 Hanting Zhang. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Hanting Zhang, Johan Commelin
-/
import tactic
import data.mv_polynomial.rename
import data.mv_polynomial.comm_ring
import algebra.algebra.subalgebra
Expand Down
1 change: 1 addition & 0 deletions src/ring_theory/witt_vector/structure_polynomial.lean
Expand Up @@ -9,6 +9,7 @@ import field_theory.mv_polynomial
import field_theory.finite.polynomial
import number_theory.basic
import ring_theory.witt_vector.witt_polynomial
import tactic.omega

/-!
# Witt structure polynomials
Expand Down

0 comments on commit ac1f3df

Please sign in to comment.