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
Equations
Instances For
def
Lean.Meta.throwTacticEx
{α : Type}
(tacticName : Name)
(mvarId : MVarId)
(msg? : Option MessageData := none)
:
MetaM α
Equations
- One or more equations did not get rendered due to their size.
Instances For
Get the type the given metavariable after instantiating metavariables and reducing to weak head normal form.
Equations
- mvarId.getType' = do let __do_lift ← mvarId.getType let __do_lift ← Lean.Meta.whnf __do_lift Lean.instantiateMVars __do_lift
Instances For
Equations
- Lean.Meta.saturate mvarId x = do let __discr ← (Lean.Meta.saturate.go x mvarId).run #[] match __discr with | (fst, r) => pure r.toList
Instances For
def
Lean.Meta.exactlyOne
(mvarIds : List MVarId)
(msg : MessageData := (MessageData.ofFormat ∘ format) "unexpected number of goals")
:
Equations
- Lean.Meta.exactlyOne [mvarId] msg = pure mvarId
- Lean.Meta.exactlyOne mvarIds msg = Lean.throwError msg
Instances For
def
Lean.Meta.ensureAtMostOne
(mvarIds : List MVarId)
(msg : MessageData := (MessageData.ofFormat ∘ 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.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- closed : TacticResultCNM
- noChange : TacticResultCNM
- modified (mvarId : MVarId) : 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.