Skip to content
This repository has been archived by the owner on Oct 25, 2023. It is now read-only.

chore: move Std -> Lean namespace #127

Merged
merged 1 commit into from Sep 28, 2022
Merged
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Jump to
Jump to file
Failed to load files.
Diff view
Diff view
2 changes: 1 addition & 1 deletion Lake/Build/Index.lean
Expand Up @@ -15,7 +15,7 @@ Lake build functions, which is used by Lake to build any Lake build info.
This module leverages the index to perform topologically-based recursive builds.
-/

open Std Lean
open Lean
namespace Lake

/--
Expand Down
1 change: 0 additions & 1 deletion Lake/Build/Topological.lean
Expand Up @@ -17,7 +17,6 @@ a build store.
This is called a suspending scheduler in *Build systems à la carte*.
-/

open Std
namespace Lake

/-!
Expand Down
2 changes: 1 addition & 1 deletion Lake/Config/Module.lean
Expand Up @@ -7,7 +7,7 @@ import Lake.Build.Trace
import Lake.Config.LeanLib

namespace Lake
open Std System
open Lean System

/-- A buildable Lean module of a `LeanLib`. -/
structure Module where
Expand Down
2 changes: 1 addition & 1 deletion Lake/Config/Package.lean
Expand Up @@ -12,7 +12,7 @@ import Lake.Config.Dependency
import Lake.Config.Script
import Lake.Util.DRBMap

open Std System Lean
open System Lean

namespace Lake

Expand Down
2 changes: 1 addition & 1 deletion Lake/Load/Elab.lean
Expand Up @@ -14,7 +14,7 @@ open Lean System
deriving instance BEq, Hashable for Import

/- Cache for the imported header environment of Lake configuration files. -/
initialize importEnvCache : IO.Ref (Std.HashMap (List Import) Environment) ← IO.mkRef {}
initialize importEnvCache : IO.Ref (HashMap (List Import) Environment) ← IO.mkRef {}

/-- Like `Lean.Elab.processHeader`, but using `importEnvCache`. -/
def processHeader (header : Syntax) (opts : Options) (trustLevel : UInt32)
Expand Down
2 changes: 1 addition & 1 deletion Lake/Load/Materialize.lean
Expand Up @@ -7,7 +7,7 @@ import Lake.Util.Git
import Lake.Load.Manifest
import Lake.Config.Dependency

open Std System Lean
open System Lean

namespace Lake

Expand Down
6 changes: 3 additions & 3 deletions Lake/Util/DRBMap.lean
Expand Up @@ -7,11 +7,11 @@ import Lean.Data.RBMap
import Lake.Util.Compare

namespace Lake
open Std RBNode
open Lean RBNode

/-!
This module includes a dependently typed adaption of the `Std.RBMap`
defined in `Std.Data.RBMap` module of the Lean core. Most of the code is
This module includes a dependently typed adaption of the `Lean.RBMap`
defined in `Lean.Data.RBMap` module of the Lean core. Most of the code is
copied directly from there with only minor edits.
-/

Expand Down
2 changes: 1 addition & 1 deletion Lake/Util/Name.lean
Expand Up @@ -12,7 +12,7 @@ namespace Lake

export Lean (Name NameMap)

@[inline] def NameMap.empty : NameMap α := Std.RBMap.empty
@[inline] def NameMap.empty : NameMap α := RBMap.empty

instance : ForIn m (NameMap α) (Name × α) where
forIn self init f := self.forIn init f
Expand Down
2 changes: 1 addition & 1 deletion Lake/Util/StoreInsts.lean
Expand Up @@ -7,7 +7,7 @@ import Lake.Util.DRBMap
import Lake.Util.Family
import Lake.Util.Store

open Std Lean
open Lean
namespace Lake

instance [Monad m] [EqOfCmpWrt κ β cmp] : MonadDStore κ β (StateT (DRBMap κ β cmp) m) where
Expand Down