Return some c
if e
is a casesOn
application.
Equations
- One or more equations did not get rendered due to their size.
Convert c
back to Expr
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.CasesOnApp.addArg
(c : Lean.Meta.CasesOnApp)
(arg : Lean.Expr)
(checkIfRefined : optParam Bool false)
:
Given a casesOn
application c
of the form
casesOn As (fun is x => motive[i, xs]) is major (fun ys_1 => (alt_1 : motive (C_1[ys_1])) ... (fun ys_n => (alt_n : motive (C_n[ys_n]) remaining
and an expression e : B[is, major]
, construct the term
casesOn As (fun is x => B[is, x] → motive[i, xs]) is major (fun ys_1 (y : B[C_1[ys_1]]) => (alt_1 : motive (C_1[ys_1])) ... (fun ys_n (y : B[C_n[ys_n]]) => (alt_n : motive (C_n[ys_n]) e remaining
We use kabstract
to abstract the is
and major
from B[is, major]
.
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.CasesOnApp.addArg.updateAlts
(c : Lean.Meta.CasesOnApp)
(checkIfRefined : optParam Bool false)
(argType : Lean.Expr)
(auxType : Lean.Expr)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.CasesOnApp.addArg?
(c : Lean.Meta.CasesOnApp)
(arg : Lean.Expr)
(checkIfRefined : optParam Bool false)
:
Similar CasesOnApp.addArg
, but returns none
on failure.
Equations
- One or more equations did not get rendered due to their size.