Equations
- One or more equations did not get rendered due to their size.
def
Lean.Compiler.LCNF.Arg.mapFVarM
{m : Type → Type}
[MonadLiftT CompilerM m]
[Monad m]
(f : FVarId → m FVarId)
(arg : Arg)
:
m Arg
Equations
- Lean.Compiler.LCNF.Arg.mapFVarM f Lean.Compiler.LCNF.Arg.erased = pure Lean.Compiler.LCNF.Arg.erased
- Lean.Compiler.LCNF.Arg.mapFVarM f (Lean.Compiler.LCNF.Arg.type e) = do let __do_lift ← Lean.Compiler.LCNF.mapFVarM f e pure ((Lean.Compiler.LCNF.Arg.type e).updateType! __do_lift)
- Lean.Compiler.LCNF.Arg.mapFVarM f (Lean.Compiler.LCNF.Arg.fvar fvarId) = do let __do_lift ← f fvarId pure ((Lean.Compiler.LCNF.Arg.fvar fvarId).updateFVar! __do_lift)
Instances For
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Compiler.LCNF.LetValue.mapFVarM
{m : Type → Type}
[MonadLiftT CompilerM m]
[Monad m]
(f : FVarId → m FVarId)
(e : LetValue)
:
m LetValue
Equations
- One or more equations did not get rendered due to their size.
- Lean.Compiler.LCNF.LetValue.mapFVarM f (Lean.Compiler.LCNF.LetValue.value value) = pure (Lean.Compiler.LCNF.LetValue.value value)
- Lean.Compiler.LCNF.LetValue.mapFVarM f Lean.Compiler.LCNF.LetValue.erased = pure Lean.Compiler.LCNF.LetValue.erased
Instances For
def
Lean.Compiler.LCNF.LetValue.forFVarM
{m : Type → Type}
[Monad m]
(f : FVarId → m Unit)
(e : LetValue)
:
m Unit
Equations
- Lean.Compiler.LCNF.LetValue.forFVarM f (Lean.Compiler.LCNF.LetValue.value value) = pure ()
- Lean.Compiler.LCNF.LetValue.forFVarM f Lean.Compiler.LCNF.LetValue.erased = pure ()
- Lean.Compiler.LCNF.LetValue.forFVarM f (Lean.Compiler.LCNF.LetValue.proj typeName idx fvarId) = f fvarId
- Lean.Compiler.LCNF.LetValue.forFVarM f (Lean.Compiler.LCNF.LetValue.const declName us args) = Array.forM (Lean.Compiler.LCNF.forFVarM f) args
- Lean.Compiler.LCNF.LetValue.forFVarM f (Lean.Compiler.LCNF.LetValue.fvar fvarId args) = do f fvarId Array.forM (Lean.Compiler.LCNF.forFVarM f) args
Instances For
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Compiler.LCNF.LetDecl.forFVarM
{m : Type → Type}
[Monad m]
(f : FVarId → m Unit)
(decl : LetDecl)
:
m Unit
Equations
- Lean.Compiler.LCNF.LetDecl.forFVarM f decl = do Lean.Compiler.LCNF.Expr.forFVarM f decl.type Lean.Compiler.LCNF.LetValue.forFVarM f decl.value
Instances For
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Compiler.LCNF.Param.mapFVarM
{m : Type → Type u_1}
[MonadLiftT CompilerM m]
[Monad m]
(f : FVarId → m FVarId)
(param : Param)
:
m Param
Equations
- Lean.Compiler.LCNF.Param.mapFVarM f param = do let __do_lift ← Lean.Compiler.LCNF.Expr.mapFVarM f param.type liftM (param.update __do_lift)
Instances For
def
Lean.Compiler.LCNF.Param.forFVarM
{m : Type → Type u_1}
[Monad m]
(f : FVarId → m Unit)
(param : Param)
:
m Unit
Equations
- Lean.Compiler.LCNF.Param.forFVarM f param = Lean.Compiler.LCNF.Expr.forFVarM f param.type
Instances For
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
- 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.
def
Lean.Compiler.LCNF.anyFVarM
{m : Type → Type}
{α : Type}
[Monad m]
[TraverseFVar α]
(f : FVarId → m Bool)
(x : α)
:
m Bool
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Compiler.LCNF.allFVarM
{m : Type → Type}
{α : Type}
[Monad m]
[TraverseFVar α]
(f : FVarId → m Bool)
(x : α)
:
m Bool
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Compiler.LCNF.anyFVar f x = (Lean.Compiler.LCNF.anyFVarM f x).run
Instances For
Equations
- Lean.Compiler.LCNF.allFVar f x = (Lean.Compiler.LCNF.allFVarM f x).run