Documentation

Lean.Compiler.IR.Basic

@[inline]
abbrev Lean.IR.FunId:
Type
Equations
@[inline]
abbrev Lean.IR.Index:
Type
Equations
Equations
@[inline]
Equations
Equations
Equations
Equations
@[inline]
abbrev Lean.IR.MData:
Type
Equations
@[inline]
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
Equations
Equations
inductive Lean.IR.Arg:
Type
Equations
  • One or more equations did not get rendered due to their size.
@[export lean_ir_mk_var_arg]
Equations
Equations
  • One or more equations did not get rendered due to their size.
structure Lean.IR.CtorInfo:
Type
Equations
  • One or more equations did not get rendered due to their size.
Equations
@[export lean_ir_mk_ctor_expr]
def Lean.IR.mkCtorExpr (n : Lean.Name) (cidx : Nat) (size : Nat) (usize : Nat) (ssize : Nat) (ys : Array Lean.IR.Arg) :
Equations
@[export lean_ir_mk_proj_expr]
Equations
@[export lean_ir_mk_uproj_expr]
Equations
@[export lean_ir_mk_sproj_expr]
Equations
@[export lean_ir_mk_fapp_expr]
Equations
@[export lean_ir_mk_papp_expr]
Equations
@[export lean_ir_mk_app_expr]
Equations
@[export lean_ir_mk_num_expr]
Equations
Equations
@[export lean_ir_mk_param]
Equations
inductive Lean.IR.AltCore (FnBody : Type) :
Type
@[export lean_ir_mk_vdecl]
Equations
@[export lean_ir_mk_jdecl]
Equations
@[export lean_ir_mk_uset]
Equations
@[export lean_ir_mk_sset]
Equations
@[export lean_ir_mk_ret]
Equations
@[export lean_ir_mk_jmp]
Equations
@[matchPattern, inline]
Equations
@[matchPattern, inline]
Equations
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.
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
  • One or more equations did not get rendered due to their size.
@[inline]
Equations
Equations
@[inline]
Equations
@[inline]
def Lean.IR.mmodifyJPs {m : TypeType} [inst : Monad m] (bs : Array Lean.IR.FnBody) (f : Lean.IR.FnBodym Lean.IR.FnBody) :
Equations
  • One or more equations did not get rendered due to their size.
@[export lean_ir_mk_alt]
def Lean.IR.mkAlt (n : Lean.Name) (cidx : Nat) (size : Nat) (usize : Nat) (ssize : Nat) (b : Lean.IR.FnBody) :
Equations
structure Lean.IR.DeclInfo:
Type
  • If some , then declaration depends on which uses a sorry axiom.

    sorryDep? : Option Lean.Name

Extra information associated with a declaration.

Equations
Equations
Equations
Equations
Equations
Equations
Equations
  • One or more equations did not get rendered due to their size.
@[export lean_ir_mk_decl]
Equations
@[export lean_ir_mk_extern_decl]
Equations
@[export lean_ir_mk_dummy_extern_decl]
Equations
@[inline]
abbrev Lean.IR.IndexSet:
Type

Set of variable and join point names

Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
Equations
  • One or more equations did not get rendered due to their size.
@[inline]
abbrev Lean.IR.VarIdSet:
Type
Equations
Equations
  • One or more equations did not get rendered due to their size.