Get the user name of the given metavariable.
Instances For
Equations
- Lean.Meta.appendTag tag suffix = tag.modifyBase fun (x : Lean.Name) => x ++ suffix.eraseMacroScopes
Instances For
Equations
- Lean.Meta.appendTagSuffix mvarId suffix = do let tag ← mvarId.getTag mvarId.setTag (Lean.Meta.appendTag tag suffix)
Instances For
def
Lean.Meta.mkFreshExprSyntheticOpaqueMVar
(type : Lean.Expr)
(tag : Lean.Name := Lean.Name.anonymous)
:
Equations
Instances For
def
Lean.Meta.throwTacticEx
{α : Type}
(tacticName : Lean.Name)
(mvarId : Lean.MVarId)
(msg? : Option Lean.MessageData := none)
:
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Throw a tactic exception with given tactic name if the given metavariable is assigned.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Get the type the given metavariable.
Instances For
Get the type the given metavariable after instantiating metavariables and reducing to weak head normal form.
Instances For
Assign mvarId
to sorryAx
Equations
- mvarId.admit synthetic = mvarId.withContext do mvarId.checkNotAssigned `admit let mvarType ← mvarId.getType let val ← Lean.Meta.mkSorry mvarType synthetic mvarId.assign val
Instances For
Beta reduce the metavariable type head
Equations
- mvarId.headBetaType = do let __do_lift ← mvarId.getType mvarId.setType __do_lift.headBeta
Instances For
Collect nondependent hypotheses that are propositions.
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Meta.saturate
(mvarId : Lean.MVarId)
(x : Lean.MVarId → Lean.MetaM (Option (List Lean.MVarId)))
:
Instances For
partial def
Lean.Meta.saturate.go
(x : Lean.MVarId → Lean.MetaM (Option (List Lean.MVarId)))
(mvarId : Lean.MVarId)
:
def
Lean.Meta.exactlyOne
(mvarIds : List Lean.MVarId)
(msg : Lean.MessageData := (Lean.MessageData.ofFormat ∘ Lean.format) "unexpected number of goals")
:
Instances For
def
Lean.Meta.ensureAtMostOne
(mvarIds : List Lean.MVarId)
(msg : Lean.MessageData := (Lean.MessageData.ofFormat ∘ Lean.format) "unexpected number of goals")
:
Equations
- Lean.Meta.ensureAtMostOne [] msg = pure none
- Lean.Meta.ensureAtMostOne [mvarId] msg = pure (some mvarId)
- Lean.Meta.ensureAtMostOne mvarIds msg = Lean.throwError msg
Instances For
Return all propositions in the local context.
Instances For
- closed: Lean.Meta.TacticResultCNM
- noChange: Lean.Meta.TacticResultCNM
- modified: Lean.MVarId → Lean.Meta.TacticResultCNM
Instances For
Check if a goal is of a subsingleton type.
Equations
- One or more equations did not get rendered due to their size.