@[inline]
Equations
- visitedConsts : Lean.NameHashSet
@[inline]
Equations
- One or more equations did not get rendered due to their size.
unsafe def
Lean.Expr.FoldConstsImpl.fold
{α : Type}
(f : Lean.Name → α → α)
(size : USize)
(e : Lean.Expr)
(acc : α)
:
Equations
- Lean.Expr.FoldConstsImpl.fold f size e acc = Lean.Expr.FoldConstsImpl.fold.visit f size e acc
unsafe def
Lean.Expr.FoldConstsImpl.fold.visit
{α : Type}
(f : Lean.Name → α → α)
(size : USize)
(e : Lean.Expr)
(acc : α)
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Expr.FoldConstsImpl.initCache = { visitedTerms := mkArray (USize.toNat Lean.Expr.FoldConstsImpl.cacheSize) (cast Lean.Expr.FoldConstsImpl.initCache.proof_1 ()), visitedConsts := ∅ }
@[inline]
unsafe def
Lean.Expr.FoldConstsImpl.foldUnsafe
{α : Type}
(e : Lean.Expr)
(init : α)
(f : Lean.Name → α → α)
:
α
@[implementedBy Lean.Expr.FoldConstsImpl.foldUnsafe]
Apply f
to every constant occurring in e
once.
Equations
- Lean.Expr.getUsedConstants e = Lean.Expr.foldConsts e #[] fun c cs => Array.push cs c
Equations
- One or more equations did not get rendered due to their size.