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.
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.expandExplicitBindersAux
(combinator : Lean.Syntax)
(idents : Array Lean.Syntax)
(type? : Option Lean.Syntax)
(body : Lean.Syntax)
:
Equations
- Lean.expandExplicitBindersAux combinator idents type? body = Lean.expandExplicitBindersAux.loop combinator idents type? (Array.size idents) body
def
Lean.expandExplicitBindersAux.loop
(combinator : Lean.Syntax)
(idents : Array Lean.Syntax)
(type? : Option Lean.Syntax)
(i : Nat)
(acc : Lean.Syntax)
:
Equations
- One or more equations did not get rendered due to their size.
- Lean.expandExplicitBindersAux.loop combinator idents type? 0 acc = pure acc
def
Lean.expandBrackedBindersAux
(combinator : Lean.Syntax)
(binders : Array Lean.Syntax)
(body : Lean.Syntax)
:
Equations
- Lean.expandBrackedBindersAux combinator binders body = Lean.expandBrackedBindersAux.loop combinator binders (Array.size binders) body
def
Lean.expandBrackedBindersAux.loop
(combinator : Lean.Syntax)
(binders : Array Lean.Syntax)
(i : Nat)
(acc : Lean.Syntax)
:
Equations
- One or more equations did not get rendered due to their size.
- Lean.expandBrackedBindersAux.loop combinator binders 0 acc = pure acc
def
Lean.expandExplicitBinders
(combinatorDeclName : Lean.Name)
(explicitBinders : Lean.Syntax)
(body : Lean.Syntax)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.expandBrackedBinders
(combinatorDeclName : Lean.Name)
(bracketedExplicitBinders : Lean.Syntax)
(body : Lean.Syntax)
:
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.
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.
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.
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.
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.
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.
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.
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.
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.
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.
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.
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.
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.
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.
Equations
- One or more equations did not get rendered due to their size.
Apply function extensionality and introduce new hypotheses.
The tactic funext
will keep applying new the funext
lemma until the goal target is not reducible to
|- ((fun x => ...) = (fun x => ...))
The variant funext h₁ ... hₙ
applies funext
n
times, and uses the given identifiers to name the new hypotheses.
Patterns can be used like in the intro
tactic. Example, given a goal
|- ((fun x : Nat × Bool => ...) = (fun x => ...))
funext (a, b)
applies funext
once and performs pattern matching on the newly introduced pair.
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.
· tac
focuses on the main goal and tries to solve it using tac
, or else fails.
Equations
- One or more equations did not get rendered due to their size.
Similar to first
, but succeeds only if one the given tactics solves the current goal.
Equations
- One or more equations did not get rendered due to their size.
@[inline]
Equations
- Lean.Loop.forIn x init f = Lean.Loop.forIn.loop f init
@[specialize]
partial def
Lean.Loop.forIn.loop
{β : Type u}
{m : Type u → Type v}
[inst : Monad m]
(f : Unit → β → m (ForInStep β))
(b : β)
:
m β
Equations
- Lean.doElemRepeat_ = Lean.ParserDescr.node `Lean.doElemRepeat_ 1022 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol "repeat ") (Lean.ParserDescr.const `doSeq))
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.
Equations
- One or more equations did not get rendered due to their size.