Skip to content

Commit

Permalink
shake
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Sep 11, 2024
1 parent 42050b8 commit 9405e9a
Show file tree
Hide file tree
Showing 5 changed files with 1 addition and 4 deletions.
1 change: 0 additions & 1 deletion Mathlib/Algebra/CharZero/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
-/
import Mathlib.Data.Int.Cast.Defs
import Mathlib.Algebra.NeZero
import Mathlib.Logic.Function.Basic

/-!
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Algebra/Order/ZeroLEOne.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jeremy Avigad, Leonardo de Moura, Mario Carneiro, Johannes Hölzl
-/
import Mathlib.Order.Basic
import Mathlib.Algebra.NeZero

/-!
# Typeclass expressing `0 ≤ 1`.
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Data/Nat/Bitwise.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,7 @@ import Mathlib.Algebra.Ring.Nat
import Mathlib.Order.Basic
import Mathlib.Tactic.AdaptationNote
import Mathlib.Tactic.Common
import Mathlib.Algebra.NeZero

/-!
# Bitwise operations on natural numbers
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Data/Nat/Cast/NeZero.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Gabriel Ebner
-/
import Mathlib.Data.Nat.Cast.Defs
import Mathlib.Algebra.NeZero

/-!
# Lemmas about nonzero elements of an `AddMonoidWithOne`
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Data/PNat/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2017 Microsoft Corporation. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Neil Strickland
-/
import Mathlib.Algebra.NeZero
import Mathlib.Data.Nat.Defs
import Mathlib.Order.Basic
import Mathlib.Order.TypeTags
Expand Down

0 comments on commit 9405e9a

Please sign in to comment.