- visited : Lean.PtrSet Lean.Expr
- counters : Lean.NameMap Nat
Instances For
@[reducible, inline]
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Expr.NumApps.main e = match StateT.run (Lean.Expr.NumApps.visit e) { visited := Lean.mkPtrSet, counters := ∅ } with | (fst, s) => s.counters
Instances For
Returns the number of applications for each declaration used in e
.
This operation is performed in IO
because the result depends on the memory representation of the object.
Note: Use this function primarily for diagnosing performance issues.
Equations
- One or more equations did not get rendered due to their size.