@[reducible, inline]
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Compiler.LCNF.PP.getFunType ps type = Lean.Compiler.LCNF.instantiateForall type (Array.map (fun (x : Lean.Compiler.LCNF.Param) => Lean.mkFVar x.fvarId) ps)
Instances For
Equations
- Lean.Compiler.LCNF.PP.run x = Lean.withOptions (fun (x : Lean.Options) => Lean.Option.set x Lean.pp.sanitizeNames false) do let __do_lift ← get ReaderT.run x __do_lift.lctx.toLocalContext
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Compiler.LCNF.ppFunDecl decl = Lean.Compiler.LCNF.PP.run do let __do_lift ← Lean.Compiler.LCNF.PP.ppFunDecl decl pure (Std.format "fun " ++ Std.format __do_lift ++ Std.format "")
Instances For
def
Lean.Compiler.LCNF.runCompilerWithoutModifyingState
{α : Type}
(x : Lean.Compiler.LCNF.CompilerM α)
 :
Execute x in CoreM without modifying Cores state.
This is useful if we want make sure we do not affect the next free variable id.
Equations
- Lean.Compiler.LCNF.runCompilerWithoutModifyingState x = do let s ← get tryFinally (x.run { lctx := { params := ∅, letDecls := ∅, funDecls := ∅ }, nextIdx := 1 }) (set s)
Instances For
Similar to ppDecl, but in CoreM, and it does not assume
decl has already been internalized.
This function is used for debugging purposes.
Equations
- Lean.Compiler.LCNF.ppDecl' decl = Lean.Compiler.LCNF.runCompilerWithoutModifyingState do let __do_lift ← decl.internalize Lean.Compiler.LCNF.ppDecl __do_lift
Instances For
Similar to ppCode, but in CoreM, and it does not assume
code has already been internalized.
Equations
- Lean.Compiler.LCNF.ppCode' code = Lean.Compiler.LCNF.runCompilerWithoutModifyingState do let __do_lift ← code.internalize Lean.Compiler.LCNF.ppCode __do_lift