Documentation

Lean.Meta.Tactic.Grind.Main

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 Lean.Meta.Grind.GrindM.run {α : Type} (x : GrindM α) (params : Params) (evalTactic? : Option EvalTactic := none) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          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 Lean.Meta.Grind.GrindM.runAtGoal {α : Type} (mvarId : MVarId) (params : Params) (k : GoalGrindM α) (evalTactic? : Option EvalTactic := none) :
                Equations
                Instances For
                  def Lean.Meta.Grind.main (mvarId : MVarId) (params : Params) :
                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    def Lean.Meta.Grind.withProtectedMCtx {m : TypeType} {α : Type} [Monad m] [MonadControlT MetaM m] [MonadLiftT MetaM m] [MonadExcept Exception m] [MonadRuntimeException m] (abstractProof : Bool) (mvarId : MVarId) (k : MVarIdm α) :
                    m α

                    A helper combinator for executing a grind-based terminal tactic. Given an input goal mvarId, it first abstracts meta-variables, cleans up local hypotheses corresponding to internal details, creates an auxiliary meta-variable mvarId', and executes k mvarId'. The execution is performed in a new meta-variable context depth to ensure that universe meta-variables cannot be accidentally assigned by grind. If k fails, it admits the input goal.

                    See issue #11806 for a motivating example.

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