@[inline]
Equations
- Lean.Meta.testHelper e p = do let __do_lift ← p e if __do_lift = true then pure true else do let __do_lift ← Lean.Meta.whnf e p __do_lift
Instances For
@[inline]
def
Lean.Meta.matchHelper?
{α : Type}
(e : Lean.Expr)
(p? : Lean.Expr → Lean.MetaM (Option α))
:
Lean.MetaM (Option α)
Instances For
Matches e
with lhs = (rhs : α)
and returns (α, lhs, rhs)
.
Instances For
Return some (α, lhs, rhs)
if e
is of the form @Eq α lhs rhs
or @HEq α lhs α rhs
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.