Equations
- Lake.instToTextModule = { toText := fun (x : Lake.Module) => x.name.toString }
Equations
- Lake.instToJsonModule = { toJson := fun (x : Lake.Module) => Lean.toJson x.name }
Equations
- Lake.instHashableModule = { hash := fun (m : Lake.Module) => hash m.keyName }
Equations
- Lake.instBEqModule = { beq := fun (m n : Lake.Module) => m.keyName == n.keyName }
@[reducible, inline]
Equations
Instances For
@[reducible, inline]
Equations
Instances For
@[inline]
Instances For
@[reducible, inline]
Equations
- Lake.ModuleMap α = Lean.RBMap Lake.Module α fun (x1 x2 : Lake.Module) => x1.name.quickCmp x2.name
Instances For
@[inline]
Equations
Instances For
Locate the named, buildable module in the library (which implies it is local and importable).
Equations
Instances For
Returns the buildable module in the library whose source file is path
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Locate the named, buildable, importable, local module in the package.
Equations
- Lake.Package.findModule? mod self = Array.findSomeRev? (fun (x : Lake.LeanLib) => Lake.LeanLib.findModule? mod x) self.leanLibs
Instances For
The library's buildable root modules.
Equations
- self.rootModules = Array.filterMap (fun (mod : Lean.Name) => Lake.LeanLib.findModule? mod self) self.config.roots
Instances For
@[inline]
Instances For
@[inline]
Equations
- Lake.Module.filePath dir ext self = Lean.modToFilePath dir self.name ext
Instances For
@[inline]
Equations
- Lake.Module.srcPath ext self = Lake.Module.filePath self.lib.srcDir ext self
Instances For
@[inline]
Equations
- Lake.Module.leanLibPath ext self = Lake.Module.filePath self.pkg.leanLibDir ext self
Instances For
@[inline]
Equations
- Lake.Module.irPath ext self = Lake.Module.filePath self.pkg.irDir ext self
Instances For
Suffix for single module dynlibs (e.g., for precompilation).
Equations
Instances For
@[inline]
Equations
- self.dynlibFile = self.pkg.leanLibDir / { toString := toString "" ++ toString self.dynlibName ++ toString "." ++ toString Lake.sharedLibExt ++ toString "" }
Instances For
@[inline]
Instances For
@[inline]
Instances For
@[inline]
Equations
- self.nativeFacets shouldExport = self.lib.nativeFacets shouldExport
Instances For
Trace Helpers #
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lake.Module.instGetMTime = { getMTime := Lake.Module.getMTime }
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lake.Module.instCheckExists = { checkExists := Lake.Module.checkExists }