Skip to content

Commit

Permalink
shake
Browse files Browse the repository at this point in the history
  • Loading branch information
Ruben-VandeVelde committed May 6, 2024
1 parent 3ddddc4 commit d297310
Show file tree
Hide file tree
Showing 4 changed files with 0 additions and 4 deletions.
1 change: 0 additions & 1 deletion Mathlib/Data/Array/ExtractLemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2024 Jiecheng Zhao. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jiecheng Zhao
-/
import Std.Data.Array.Lemmas
/-!
# Lemmas about `Array.extract`
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Data/List/EditDistance/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: Kim Liesinger
-/
import Mathlib.Algebra.Group.Defs
import Std.Data.List.Lemmas

/-!
# Levenshtein distances
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Data/UnionFind.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Mario Carneiro
-/
import Mathlib.Init.Data.Nat.Lemmas
import Mathlib.Init.Order.LinearOrder
import Std.Data.Array.Lemmas

set_option autoImplicit true

Expand Down
1 change: 0 additions & 1 deletion Mathlib/Init/Data/List/Instances.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2016 Microsoft Corporation. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Leonardo de Moura
-/
import Std.Data.List.Lemmas
import Mathlib.Mathport.Rename

#align_import init.data.list.instances from "leanprover-community/lean"@"9af482290ef68e8aaa5ead01aa7b09b7be7019fd"
Expand Down

0 comments on commit d297310

Please sign in to comment.