- header : String
- opts : Lean.Options
- currNamespace : Lean.Name
- openDecls : List Lean.OpenDecl
section variables
varDecls : Array (Lean.TSyntax `Lean.Parser.Term.bracketedBinder)Globally unique internal identifiers for the
varDecls
noncomputable sections automatically add the
noncomputable
modifier to any declaration we cannot generate code for.isNoncomputable : Bool
Equations
- One or more equations did not get rendered due to their size.
- env : Lean.Environment
- messages : Lean.MessageLog
- scopes : List Lean.Elab.Command.Scope
- nextMacroScope : Nat
- maxRecDepth : Nat
- nextInstIdx : Nat
- ngen : Lean.NameGenerator
- infoState : Lean.Elab.InfoState
- traceState : Lean.TraceState
Equations
- One or more equations did not get rendered due to their size.
- fileName : String
- fileMap : Lean.FileMap
- currRecDepth : Nat
- cmdPos : String.Pos
- macroStack : Lean.Elab.MacroStack
- currMacroScope : Lean.MacroScope
- ref : Lean.Syntax
- tacticCache? : Option (IO.Ref Lean.Elab.Tactic.Cache)
@[inline]
@[inline]
@[inline]
@[inline]
Equations
Equations
- Lean.Elab.Command.instMonadCommandElabM = let i := inferInstanceAs (Monad Lean.Elab.Command.CommandElabM); Monad.mk
def
Lean.Elab.Command.mkState
(env : Lean.Environment)
(messages : optParam Lean.MessageLog
{ msgs :=
{ root := Std.PersistentArrayNode.node (Array.mkEmpty (USize.toNat Std.PersistentArray.branching)),
tail := Array.mkEmpty (USize.toNat Std.PersistentArray.branching), size := 0,
shift := Std.PersistentArray.initShift, tailOff := 0 } })
(opts : optParam Lean.Options { entries := [] })
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.addLinter l = do let ls ← ST.Ref.get Lean.Elab.Command.lintersRef ST.Ref.set Lean.Elab.Command.lintersRef (Array.push ls l)
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
- Lean.Elab.Command.instMonadOptionsCommandElabM = { getOptions := do let a ← get pure (List.head! a.scopes).opts }
Equations
- Lean.Elab.Command.getRef = do let a ← read pure a.ref
Equations
- Lean.Elab.Command.instAddMessageContextCommandElabM = { addMessageContext := Lean.addMessageContextPartial }
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.Elab.Command.mkMessageAux
(ctx : Lean.Elab.Command.Context)
(ref : Lean.Syntax)
(msgData : Lean.MessageData)
(severity : Lean.MessageSeverity)
:
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.
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Command.instMonadLiftTIOCommandElabM = { monadLift := fun {α} => Lean.Elab.Command.liftIO }
Equations
- Lean.Elab.Command.getScope = do let a ← get pure (List.head! a.scopes)
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
- Lean.Elab.Command.getCurrMacroScope = do let a ← read pure a.currMacroScope
Equations
- Lean.Elab.Command.getMainModule = do let a ← Lean.getEnv pure (Lean.Environment.mainModule a)
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Command.instMonadQuotationCommandElabM = Lean.MonadQuotation.mk Lean.Elab.Command.getCurrMacroScope Lean.Elab.Command.getMainModule fun {α} => Lean.Elab.Command.withFreshMacroScope
Equations
- One or more equations did not get rendered due to their size.
@[implementedBy Lean.Elab.Command.mkCommandElabAttributeUnsafe]
def
Lean.Elab.Command.withMacroExpansion
{α : Type}
(beforeStx : Lean.Syntax)
(afterStx : Lean.Syntax)
(x : Lean.Elab.Command.CommandElabM α)
:
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.
elabCommand
wrapper that should be used for the initial invocation, not for recursive calls after
macro expansion etc.
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Command.adaptExpander
(exp : Lean.Syntax → Lean.Elab.Command.CommandElabM Lean.Syntax)
:
Adapt a syntax transformation to a regular, command-producing elaborator.
Equations
- Lean.Elab.Command.adaptExpander exp stx = do let stx' ← exp stx Lean.Elab.Command.withMacroExpansion stx stx' (Lean.Elab.Command.elabCommand stx')
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Command.liftTermElabM
{α : Type}
(declName? : Option Lean.Name)
(x : Lean.Elab.TermElabM α)
:
Equations
- One or more equations did not get rendered due to their size.
@[inline]
def
Lean.Elab.Command.runTermElabM
{α : Type}
(declName? : Option Lean.Name)
(elabFn : Array Lean.Expr → Lean.Elab.TermElabM α)
:
Equations
- One or more equations did not get rendered due to their size.
@[inline]
Equations
- Lean.Elab.Command.catchExceptions x ctx ref = EIO.catchExceptions (Lean.Elab.Command.withLogging x ctx ref) fun x => pure ()
Equations
- Lean.Elab.Command.getScopes = do let a ← get pure a.scopes
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Command.withScope
{α : Type}
(f : Lean.Elab.Command.Scope → Lean.Elab.Command.Scope)
(x : Lean.Elab.Command.CommandElabM α)
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Command.getLevelNames = do let a ← Lean.Elab.Command.getScope pure a.levelNames
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.