@[reducible, inline]
Instances For
instance
Lean.Elab.OpenDecl.instMonadResolveNameM
{m : Type → Type}
[Monad m]
[MonadLiftT (ST IO.RealWorld) m]
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.OpenDecl.resolveId
{m : Type → Type}
[Monad m]
[MonadEnv m]
[MonadExceptOf Exception m]
[MonadRef m]
[AddMessageContext m]
[MonadLiftT (ST IO.RealWorld) m]
(ns : Name)
(idStx : Syntax)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.OpenDecl.elabOpenDecl
{m : Type → Type}
[Monad m]
[MonadEnv m]
[MonadExceptOf Exception m]
[MonadRef m]
[AddMessageContext m]
[MonadLiftT (ST IO.RealWorld) m]
[MonadLog m]
[MonadResolveName m]
[MonadInfoTree m]
(stx : TSyntax `Lean.Parser.Command.openDecl)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.OpenDecl.resolveNameUsingNamespaces
{m : Type → Type}
[Monad m]
[MonadEnv m]
[MonadExceptOf Exception m]
[MonadRef m]
[AddMessageContext m]
[MonadLiftT (ST IO.RealWorld) m]
[MonadLog m]
[MonadResolveName m]
(nss : List Name)
(idStx : Ident)
:
m Name
Equations
- One or more equations did not get rendered due to their size.