@[inline]
Equations
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Expr.FindImpl.findM? p size e = Lean.Expr.FindImpl.findM?.visit p size e
Equations
- One or more equations did not get rendered due to their size.
Equations
Return true if e
occurs in t
Equations
- Lean.Expr.occurs e t = Option.isSome (Lean.Expr.find? (fun s => s == e) t)
- found: Lean.Expr.FindStep
- visit: Lean.Expr.FindStep
- done: Lean.Expr.FindStep
Return type for findExt?
function argument.
unsafe def
Lean.Expr.FindExtImpl.findM?
(p : Lean.Expr → Lean.Expr.FindStep)
(size : USize)
(e : Lean.Expr)
:
Equations
- Lean.Expr.FindExtImpl.findM? p size e = Lean.Expr.FindExtImpl.findM?.visit p size e
unsafe def
Lean.Expr.FindExtImpl.findM?.visitApp
(p : Lean.Expr → Lean.Expr.FindStep)
(size : USize)
(e : Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
unsafe def
Lean.Expr.FindExtImpl.findM?.visit
(p : Lean.Expr → Lean.Expr.FindStep)
(size : USize)
(e : Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.