Equations
- Aesop.Rapp.runMetaM x r = r.metaState.runMetaM x
Instances For
Equations
- Aesop.Rapp.runMetaM' x r = Prod.fst <$> Aesop.Rapp.runMetaM x r
Instances For
def
Aesop.Rapp.runMetaMModifying
{α : Type}
(x : Lean.MetaM α)
(r : Aesop.Rapp)
 :
Lean.MetaM (α × Aesop.Rapp)
Equations
- Aesop.Rapp.runMetaMModifying x r = do let __discr ← Aesop.Rapp.runMetaM x r match __discr with | (result, finalState) => pure (result, Aesop.Rapp.setMetaState finalState r)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Goal.runMetaMInPostNormState
{α : Type}
(x : Lean.MVarId → Lean.MetaM α)
(g : Aesop.Goal)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.Goal.runMetaMInPostNormState'
{α : Type}
(x : Lean.MVarId → Lean.MetaM α)
(g : Aesop.Goal)
 :
Equations
- Aesop.Goal.runMetaMInPostNormState' x g = Prod.fst <$> Aesop.Goal.runMetaMInPostNormState x g
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Aesop.Goal.runMetaMInParentState' x g = Prod.fst <$> Aesop.Goal.runMetaMInParentState x g
Instances For
Equations
- Aesop.Goal.runMetaMModifyingParentState x g = do let __do_lift ← liftM g.parentRapp? match __do_lift with | none => x | some rref => Aesop.RappRef.runMetaMModifying x rref
Instances For
Equations
- Aesop.Rapp.runMetaMInParentState x r = do let __do_lift ← ST.Ref.get r.parent Aesop.Goal.runMetaMInParentState x __do_lift
Instances For
Equations
- Aesop.Rapp.runMetaMInParentState' x r = do let __do_lift ← ST.Ref.get r.parent Aesop.Goal.runMetaMInParentState' x __do_lift
Instances For
Equations
- Aesop.Rapp.runMetaMModifyingParentState x r = do let __do_lift ← ST.Ref.get r.parent Aesop.Goal.runMetaMModifyingParentState x __do_lift