- step: Lean.Name → Array Lean.IR.Decl → Lean.IR.LogEntry
- message: Lean.Format → Lean.IR.LogEntry
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.IR.LogEntry.instToFormatLogEntry = { format := Lean.IR.LogEntry.fmt }
Equations
- One or more equations did not get rendered due to their size.
@[export lean_ir_log_to_string]
Equations
@[inline]
Equations
- Lean.IR.log entry = modify fun s => { env := s.env, log := Array.push s.log entry }
Equations
- Lean.IR.tracePrefixOptionName = `trace.compiler.ir
@[inline]
Equations
- Lean.IR.logDecls cls decl = Lean.IR.logDeclsAux (Lean.IR.tracePrefixOptionName ++ cls) cls decl
@[inline]
Equations
@[inline]
@[inline]
Equations
- Lean.IR.modifyEnv f = modify fun s => { env := f s.env, log := s.log }
@[inline]
Equations
@[export lean_ir_find_env_decl]
Equations
Equations
- Lean.IR.findDecl n = do let a ← get pure (Lean.IR.findEnvDecl a.env n)
Equations
- Lean.IR.containsDecl n = do let a ← get pure (Lean.SMap.contains (Lean.SimplePersistentEnvExtension.getState Lean.IR.declMapExt a.env) n)
Equations
- One or more equations did not get rendered due to their size.
@[export lean_ir_add_decl]
Equations
- Lean.IR.addDeclAux env decl = Lean.PersistentEnvExtension.addEntry Lean.IR.declMapExt env decl
Equations
Equations
- Lean.IR.getEnv = do let s ← get pure s.env
Equations
- Lean.IR.addDecl decl = Lean.IR.modifyEnv fun env => Lean.PersistentEnvExtension.addEntry Lean.IR.declMapExt env decl
Equations
- Lean.IR.addDecls decls = Array.forM Lean.IR.addDecl decls 0 (Array.size decls)
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.IR.findDecl' n decls = do let a ← get pure (Lean.IR.findEnvDecl' a.env n decls)
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
@[export lean_decl_get_sorry_dep]
Equations
- One or more equations did not get rendered due to their size.