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
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
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[inline]
def
Aesop.MVarClusterRef.checkState.go
{σ : Type}
[BEq σ]
[ToString σ]
(id : String)
(expected : σ)
(actual : σ)
 :
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
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.MVarClusterRef.checkMVars
(root : Aesop.MVarClusterRef)
(rootMetaState : Lean.Meta.SavedState)
 :
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
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
def
Aesop.MVarClusterRef.checkMVars.checkGoalMVars
(rootMetaState : Lean.Meta.SavedState)
(g : Aesop.Goal)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.MVarClusterRef.checkMVars.checkNormMVars
(rootMetaState : Lean.Meta.SavedState)
(g : Aesop.Goal)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.MVarClusterRef.checkIntroducedMVars
(root : Aesop.MVarClusterRef)
(rootMetaState : Lean.Meta.SavedState)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.MVarClusterRef.checkInvariants
(root : Aesop.MVarClusterRef)
(rootMetaState : Lean.Meta.SavedState)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.MVarClusterRef.checkInvariantsIfEnabled
(root : Aesop.MVarClusterRef)
(rootMetaState : Lean.Meta.SavedState)
 :
Equations
- root.checkInvariantsIfEnabled rootMetaState = do let __do_lift ← Aesop.Check.tree.isEnabled if __do_lift = true then root.checkInvariants rootMetaState else pure PUnit.unit
Instances For
Equations
- Aesop.checkInvariantsIfEnabled = do let __do_lift ← Aesop.getRootMVarCluster let __do_lift_1 ← Aesop.getRootMetaState liftM (__do_lift.checkInvariantsIfEnabled __do_lift_1)