Instances For
@[inline]
Equations
Instances For
Equations
- Lean.Meta.Grind.AC.checkMaxSteps = do let __do_lift ← Lean.Meta.Grind.AC.get' let __do_lift_1 ← liftM Lean.Meta.Grind.getConfig pure (decide (__do_lift.steps ≥ __do_lift_1.acSteps))
Instances For
Equations
- Lean.Meta.Grind.AC.incSteps = Lean.Meta.Grind.AC.modify' fun (s : Lean.Meta.Grind.AC.State) => { structs := s.structs, opIdOf := s.opIdOf, exprToOpIds := s.exprToOpIds, steps := s.steps + 1 }
Instances For
@[always_inline]
instance
Lean.Meta.Grind.AC.instMonadGetStructOfMonadLift
(m n : Type → Type)
[MonadLift m n]
[MonadGetStruct m]
:
Equations
- Lean.Meta.Grind.AC.instMonadGetStructOfMonadLift m n = { getStruct := liftM Lean.Meta.Grind.AC.getStruct }
@[reducible, inline]
Instances For
@[reducible, inline]
Equations
- Lean.Meta.Grind.AC.getOpId = do let __do_lift ← read pure __do_lift.opId
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Equations
- Lean.Meta.Grind.AC.getOp = do let __do_lift ← Lean.Meta.Grind.AC.getStruct pure __do_lift.op
Instances For
Equations
- Lean.Meta.Grind.AC.getTermOpIds e = do let __do_lift ← Lean.Meta.Grind.AC.get' pure ((Lean.PersistentHashMap.find? __do_lift.exprToOpIds { expr := e }).getD [])
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
- Lean.Meta.Grind.AC.isCommutative = do let __do_lift ← Lean.Meta.Grind.AC.getStruct pure __do_lift.commInst?.isSome
Instances For
Equations
- Lean.Meta.Grind.AC.hasNeutral = do let __do_lift ← Lean.Meta.Grind.AC.getStruct pure __do_lift.neutralInst?.isSome
Instances For
Equations
- Lean.Meta.Grind.AC.isIdempotent = do let __do_lift ← Lean.Meta.Grind.AC.getStruct pure __do_lift.idempotentInst?.isSome