Skip to content

Commit

Permalink
chore: fix imports (#8538)
Browse files Browse the repository at this point in the history
  • Loading branch information
fgdorais committed Nov 20, 2023
1 parent 43b4712 commit f659b7b
Show file tree
Hide file tree
Showing 8 changed files with 9 additions and 8 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Field/Defs.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Robert Lewis, Leonardo de Moura, Johannes Hölzl, Mario Carneiro
-/

import Mathlib.Algebra.Ring.Defs
import Std.Data.Rat
import Std.Data.Rat.Basic
import Mathlib.Data.Rat.Init

#align_import algebra.field.defs from "leanprover-community/mathlib"@"2651125b48fc5c170ab1111afd0817c903b1fc6c"
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Data/HashMap.lean
Expand Up @@ -8,8 +8,8 @@ nothing from the mathlib3 file `data.hash_map` is reflected here.
The porting header is just here to mark that no further work on `data.hash_map` is desired.
-/
import Mathlib.Init.Align
import Std.Data.HashMap
import Std.Data.RBMap
import Std.Data.HashMap.Basic
import Std.Data.RBMap.Basic

#align_import data.hash_map from "leanprover-community/mathlib"@"f0c8bf9245297a541f468be517f1bde6195105e9"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/MLList/Dedup.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import Std.Data.MLList.Basic
import Std.Data.HashMap
import Std.Data.HashMap.Basic

/-!
# Lazy deduplication of lazy lists
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Rat/Init.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Mario Carneiro
-/
import Mathlib.Mathport.Rename
import Std.Data.Rat
import Std.Data.Rat.Basic

#align_import data.rat.init from "leanprover-community/mathlib"@"f340f229b1f461aa1c8ee11e0a172d0a3b301a4a"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Tree.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2019 mathlib community. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Wojciech Nawrocki
-/
import Std.Data.RBMap
import Std.Data.RBMap.Basic
import Mathlib.Data.Num.Basic
import Mathlib.Order.Basic
import Mathlib.Init.Data.Ordering.Basic
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Lean/Data/NameMap.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jon Eugster
-/
import Lean.Data.NameMap
import Std.Data.RBMap
import Std.Data.RBMap.Basic

/-!
# Additional functions on `Lean.NameMap`.
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Lean/Name.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2023 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import Std.Data.HashMap
import Std.Data.HashMap.Basic
import Mathlib.Lean.SMap
import Mathlib.Lean.Expr.Basic

Expand Down
1 change: 1 addition & 0 deletions Mathlib/Util/LongNames.lean
Expand Up @@ -3,6 +3,7 @@ Copyright (c) 2023 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import Std.Data.HashMap.WF
import Mathlib.Lean.Name
import Mathlib.Lean.Expr.Basic

Expand Down

0 comments on commit f659b7b

Please sign in to comment.