def
Lean.Elab.Tactic.elabTerm
(stx : Lean.Syntax)
(expectedType? : Option Lean.Expr)
(mayPostpone : optParam Bool false)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Tactic.elabTerm.go
(stx : Lean.Syntax)
(expectedType? : Option Lean.Expr)
(mayPostpone : optParam Bool false)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Tactic.elabTermEnsuringType
(stx : Lean.Syntax)
(expectedType? : Option Lean.Expr)
(mayPostpone : optParam Bool false)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Tactic.closeMainGoalUsing
(x : Lean.Expr → Lean.Elab.Tactic.TacticM Lean.Expr)
(checkUnassigned : optParam Bool true)
:
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Elab.Tactic.logUnassignedAndAbort mvarIds = do let a ← liftM (Lean.Elab.Term.logUnassignedUsingErrorInfos mvarIds none) if a = true then Lean.Elab.throwAbortTactic else pure PUnit.unit
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.Elab.Tactic.elabTermWithHoles
(stx : Lean.Syntax)
(expectedType? : Option Lean.Expr)
(tagSuffix : Lean.Name)
(allowNaturalHoles : optParam Bool false)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Tactic.refineCore
(stx : Lean.Syntax)
(tagSuffix : Lean.Name)
(allowNaturalHoles : Bool)
:
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.
Given a tactic
apply f
we want the apply
tactic to create all metavariables. The following
definition will return @f
for f
. That is, it will not create
metavariables for implicit arguments.
A similar method is also used in Lean 3.
This method is useful when applying lemmas such as:
theorem infLeRight {s t : Set α} : s ⊓ t ≤ t
where s ≤ t
here is defined as
∀ {x : α}, x ∈ s → x ∈ t
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.Tactic.evalApplyLikeTactic
(tac : Lean.MVarId → Lean.Expr → Lean.MetaM (List Lean.MVarId))
(e : 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.
def
Lean.Elab.Tactic.elabAsFVar
(stx : Lean.Syntax)
(userName? : optParam (Option Lean.Name) none)
:
Elaborate stx
. If it a free variable, return it. Otherwise, assert it, and return the free variable.
Note that, the main goal is updated when Meta.assert
is used in the second case.
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.