Skip to content

Commit

Permalink
chore: import cleanup in Init (#6522)
Browse files Browse the repository at this point in the history
This PR avoids unnecessarily importing "kitchen sink" files.
  • Loading branch information
kim-em authored Jan 4, 2025
1 parent cdeb958 commit 9080df3
Show file tree
Hide file tree
Showing 9 changed files with 5 additions and 8 deletions.
1 change: 0 additions & 1 deletion src/Lean/Data/Lsp/Utf16.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,6 @@ Authors: Marc Huisinga, Wojciech Nawrocki
-/
prelude
import Init.Data.String
import Init.Data.Array
import Lean.Data.Lsp.Basic
import Lean.Data.Position
import Lean.DeclarationRange
Expand Down
1 change: 1 addition & 0 deletions src/Lean/Linter/MissingDocs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
-/
prelude
import Lean.Parser.Syntax
import Lean.Meta.Tactic.Simp.RegisterCommand
import Lean.Elab.Command
import Lean.Elab.SetOption
Expand Down
1 change: 0 additions & 1 deletion src/Lean/PrettyPrinter/Delaborator/Builtins.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: Sebastian Ullrich, Leonardo de Moura, Gabriel Ebner, Mario Carneiro
-/
prelude
import Lean.Parser
import Lean.PrettyPrinter.Delaborator.Attributes
import Lean.PrettyPrinter.Delaborator.Basic
import Lean.PrettyPrinter.Delaborator.SubExpr
Expand Down
1 change: 1 addition & 0 deletions src/Lean/Server/Completion.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,6 +5,7 @@ Authors: Leonardo de Moura, Marc Huisinga
-/
prelude
import Lean.Server.Completion.CompletionCollectors
import Std.Data.HashMap

namespace Lean.Server.Completion
open Lsp
Expand Down
4 changes: 2 additions & 2 deletions src/Lean/Util/ShareCommon.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,8 +5,8 @@ Authors: Leonardo de Moura
-/
prelude
import Init.ShareCommon
import Std.Data.HashSet
import Std.Data.HashMap
import Std.Data.HashSet.Basic
import Std.Data.HashMap.Basic
import Lean.Data.PersistentHashMap
import Lean.Data.PersistentHashSet

Expand Down
1 change: 0 additions & 1 deletion src/Std/Sat/AIG/Basic.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: Henrik Böving
-/
prelude
import Std.Data.HashMap
import Std.Data.HashSet

namespace Std
Expand Down
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: Josh Clune
-/
prelude
import Init.Data.Array
import Std.Tactic.BVDecide.LRAT.Internal.Formula.Class
import Std.Tactic.BVDecide.LRAT.Internal.Assignment
import Std.Sat.CNF.Basic
Expand Down
1 change: 0 additions & 1 deletion src/Std/Time/DateTime/Timestamp.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Sofia Rodrigues
-/
prelude
import Std.Time.Internal
import Init.Data.Int
import Init.System.IO
import Std.Time.Time
import Std.Time.Date
Expand Down
2 changes: 1 addition & 1 deletion src/Std/Time/Internal/Bounded.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Sofia Rodrigues
-/
prelude
import Init.Data.Int
import Init.Omega

namespace Std
namespace Time
Expand Down

0 comments on commit 9080df3

Please sign in to comment.