- step: Lean.Name → Array Lean.IR.Decl → Lean.IR.LogEntry
- message: Lean.Format → Lean.IR.LogEntry
Instances For
Equations
- One or more equations did not get rendered due to their size.
- (Lean.IR.LogEntry.message msg).fmt = msg
Instances For
Equations
- Lean.IR.LogEntry.instToFormat = { format := Lean.IR.LogEntry.fmt }
@[reducible, inline]
Instances For
Equations
- Lean.IR.log entry = modify fun (s : Lean.IR.CompilerState) => { env := s.env, log := Array.push s.log entry }
Instances For
Equations
- Lean.IR.tracePrefixOptionName = `trace.compiler.ir
Instances For
@[inline]
Instances For
@[inline]
Equations
Instances For
@[inline]
Instances For
@[inline]
Equations
- Lean.IR.modifyEnv f = modify fun (s : Lean.IR.CompilerState) => { env := f s.env, log := s.log }
Instances For
@[export lean_ir_find_env_decl]
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[export lean_ir_add_decl]
Instances For
Equations
- Lean.IR.getEnv = do let s ← get pure s.env
Instances For
Instances For
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[export lean_decl_get_sorry_dep]
Equations
- Lean.IR.getSorryDep env declName = match Lean.IR.findEnvDecl env declName with | some (Lean.IR.Decl.fdecl f xs type body { sorryDep? := dep? }) => dep? | x => none