Documentation

Lean.Meta.Tactic.Grind.Arith.CommRing.MonadRing

  • canonExpr : Exprm Expr

    Helper function for removing dependency on GoalM. In RingM and SemiringM, this is just sharedCommon (← canon e) When printing counterexamples, we are at MetaM, and this is just the identity function.

  • synthInstance? : Exprm (Option Expr)

    Helper function for removing dependency on GoalM. During search we want to track the instances synthesized by grind, and this is Grind.synthInstance.

Instances
    @[always_inline]
    Equations
    • One or more equations did not get rendered due to their size.
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      Instances
        @[always_inline]
        Equations
        • One or more equations did not get rendered due to their size.
        Instances
          @[always_inline]
          Equations
          • One or more equations did not get rendered due to their size.
          @[always_inline]
          Equations
          • One or more equations did not get rendered due to their size.