Equations
- Lean.Meta.Match.mkNamedPattern x h p = Lean.Meta.mkAppM `namedPattern #[x, p, h]
Equations
- One or more equations did not get rendered due to their size.
- inaccessible: Lean.Expr → Lean.Meta.Match.Pattern
- var: Lean.FVarId → Lean.Meta.Match.Pattern
- ctor: Lean.Name → List Lean.Level → List Lean.Expr → List Lean.Meta.Match.Pattern → Lean.Meta.Match.Pattern
- val: Lean.Expr → Lean.Meta.Match.Pattern
- arrayLit: Lean.Expr → List Lean.Meta.Match.Pattern → Lean.Meta.Match.Pattern
- as: Lean.FVarId → Lean.Meta.Match.Pattern → Lean.FVarId → Lean.Meta.Match.Pattern
Equations
- Lean.Meta.Match.instInhabitedPattern = { default := Lean.Meta.Match.Pattern.inaccessible default }
Equations
- Lean.Meta.Match.Pattern.toExpr p annotate = Lean.Meta.Match.Pattern.toExpr.visit annotate p
partial def
Lean.Meta.Match.Pattern.toExpr.visit
(annotate : optParam Bool false)
(p : Lean.Meta.Match.Pattern)
:
def
Lean.Meta.Match.Pattern.replaceFVarId
(fvarId : Lean.FVarId)
(v : Lean.Expr)
(p : Lean.Meta.Match.Pattern)
:
Equations
- Lean.Meta.Match.Pattern.replaceFVarId fvarId v p = let s := { map := ∅ }; Lean.Meta.Match.Pattern.applyFVarSubst (Lean.Meta.FVarSubst.insert s fvarId v) p
- ref : Lean.Syntax
- fvarDecls : List Lean.LocalDecl
- patterns : List Lean.Meta.Match.Pattern
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
- ref : Lean.Syntax
- idx : Nat
- rhs : Lean.Expr
- fvarDecls : List Lean.LocalDecl
- patterns : List Lean.Meta.Match.Pattern
Equations
- Lean.Meta.Match.instInhabitedAlt = { default := { ref := default, idx := default, rhs := default, fvarDecls := default, patterns := default } }
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.Match.Alt.replaceFVarId
(fvarId : Lean.FVarId)
(v : Lean.Expr)
(alt : Lean.Meta.Match.Alt)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.Match.Alt.checkAndReplaceFVarId
(fvarId : Lean.FVarId)
(v : Lean.Expr)
(alt : Lean.Meta.Match.Alt)
:
Equations
- One or more equations did not get rendered due to their size.
- var: Lean.FVarId → Lean.Meta.Match.Example
- underscore: Lean.Meta.Match.Example
- ctor: Lean.Name → List Lean.Meta.Match.Example → Lean.Meta.Match.Example
- val: Lean.Expr → Lean.Meta.Match.Example
- arrayLit: List Lean.Meta.Match.Example → Lean.Meta.Match.Example
partial def
Lean.Meta.Match.Example.replaceFVarId
(fvarId : Lean.FVarId)
(ex : Lean.Meta.Match.Example)
:
Equations
- One or more equations did not get rendered due to their size.
- mvarId : Lean.MVarId
- alts : List Lean.Meta.Match.Alt
- examples : List Lean.Meta.Match.Example
Equations
- Lean.Meta.Match.instInhabitedProblem = { default := { mvarId := default, vars := default, alts := default, examples := default } }
Equations
- Lean.Meta.Match.withGoalOf p x = Lean.Meta.withMVarContext p.mvarId x
Equations
- One or more equations did not get rendered due to their size.
@[inline]
- matcher : Lean.Expr
- counterExamples : List Lean.Meta.Match.CounterExample
- addMatcher : Lean.MetaM Unit