- info : ConstantInfo
- kind : MetaM Lsp.CompletionItemKind
Instances For
@[reducible, inline]
Equations
Instances For
Cached header declarations for which allowCompletion headerEnv decl
is true.
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
Returns the declarations in the header for which allowCompletion env decl
is true, caching them
if not already cached.
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.Completion.forEligibleDeclsM
{m : Type → Type}
[Monad m]
[MonadEnv m]
[MonadLiftT MetaM m]
(f : Name → EligibleDecl → m PUnit)
:
m PUnit
Iterate over all declarations that are allowed in completion results.
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Server.Completion.allowCompletion
(eligibleHeaderDecls : EligibleHeaderDecls)
(env : Environment)
(declName : Name)
:
Checks whether this declaration can appear in completion results.
Equations
- One or more equations did not get rendered due to their size.