- ite : Lean.Meta.SplitKind
- match : Lean.Meta.SplitKind
- both : Lean.Meta.SplitKind
Instances For
Equations
- Lean.Meta.SplitKind.ite.considerIte = true
- Lean.Meta.SplitKind.both.considerIte = true
- x✝.considerIte = false
Instances For
Equations
- Lean.Meta.SplitKind.match.considerMatch = true
- Lean.Meta.SplitKind.both.considerMatch = true
- x✝.considerMatch = false
Instances For
- exceptionSet : Lean.ExprSet
- kind : Lean.Meta.SplitKind
Instances For
@[reducible, inline]
Equations
Instances For
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Meta.findSplit?
(e : Lean.Expr)
(kind : Lean.Meta.SplitKind := Lean.Meta.SplitKind.both)
(exceptionSet : Lean.ExprSet := ∅)
:
Return an if-then-else
or match-expr
to split.
Equations
- Lean.Meta.findSplit? e kind exceptionSet = do let __do_lift ← Lean.instantiateMVars e Lean.Meta.findSplit?.go kind exceptionSet __do_lift
Instances For
partial def
Lean.Meta.findSplit?.go
(kind : Lean.Meta.SplitKind := Lean.Meta.SplitKind.both)
(exceptionSet : Lean.ExprSet := ∅)
(e : Lean.Expr)
:
def
Lean.Meta.findSplit?.find?
(kind : Lean.Meta.SplitKind := Lean.Meta.SplitKind.both)
(exceptionSet : Lean.ExprSet := ∅)
(e : Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Default Simp.Context
for simpIf
methods. It contains all congruence theorems, but
just the rewriting rules for reducing if
expressions.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Meta.SplitIf.mkDischarge? useDecide = do let __do_lift ← Lean.getLCtx pure (Lean.Meta.SplitIf.discharge?✝ __do_lift.numIndices useDecide)
Instances For
def
Lean.Meta.SplitIf.splitIfAt?
(mvarId : Lean.MVarId)
(e : Lean.Expr)
(hName? : Option Lean.Name)
:
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.
Instances For
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.
Instances For
def
Lean.Meta.splitIfLocalDecl?
(mvarId : Lean.MVarId)
(fvarId : Lean.FVarId)
(hName? : Option Lean.Name := none)
:
Equations
- One or more equations did not get rendered due to their size.