- spawnArgs : IO.Process.SpawnArgs
- exitCode : UInt32
- stdout : String
- stderr : String
Instances For
def
Lean.Server.FileWorker.runLakeSetupFile
(m : DocumentMeta)
(lakePath filePath : System.FilePath)
(header : ModuleHeader)
(handleStderr : String → IO Unit)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
partial def
Lean.Server.FileWorker.runLakeSetupFile.processStderr
(lakePath : System.FilePath)
(handleStderr : String → IO Unit)
(args : Array String)
(lakeProc :
IO.Process.Child
{ stdin := IO.Process.Stdio.null,
stdout :=
{ stdin := IO.Process.Stdio.piped, stdout := IO.Process.Stdio.piped, stderr := IO.Process.Stdio.piped,
cmd := lakePath.toString, args := args }.stdout,
stderr :=
{ stdin := IO.Process.Stdio.piped, stdout := IO.Process.Stdio.piped, stderr := IO.Process.Stdio.piped,
cmd := lakePath.toString, args := args }.stderr })
(acc : String)
:
Categorizes possible outcomes of running lake setup-file
.
- success : FileSetupResultKind
File configuration loaded and dependencies updated successfully.
- noLakefile : FileSetupResultKind
No Lake project found, no setup was done.
- importsOutOfDate : FileSetupResultKind
Imports must be rebuilt but
--no-build
was specified. - error
(msg : String)
: FileSetupResultKind
Other error during Lake invocation.
Instances For
Result of running lake setup-file
.
- kind : FileSetupResultKind
Kind of outcome.
- setup : ModuleSetup
Configuration from a successful setup, or else the default.
Instances For
Equations
- Lean.Server.FileWorker.FileSetupResult.ofSuccess setup = pure { kind := Lean.Server.FileWorker.FileSetupResultKind.success, setup := setup }
Instances For
def
Lean.Server.FileWorker.FileSetupResult.ofNoLakefile
(m : DocumentMeta)
(header : ModuleHeader)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.FileSetupResult.ofImportsOutOfDate
(m : DocumentMeta)
(header : ModuleHeader)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.FileSetupResult.ofError
(m : DocumentMeta)
(header : ModuleHeader)
(msg : String)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.FileWorker.setupFile
(m : DocumentMeta)
(header : ModuleHeader)
(handleStderr : String → IO Unit)
:
Uses lake setup-file
to compile dependencies on the fly and add them to LEAN_PATH
.
Compilation progress is reported to handleStderr
. Returns the search path for
source files and the options for the file.