Documentation

Lean.Meta.Tactic.Grind.Intro

def Lean.Meta.Grind.intros (goal : Goal) (generation : Nat) :

Introduce new hypotheses (and apply by_contra) until goal is of the form ... ⊢ False

Equations
Instances For
    def Lean.Meta.Grind.assertAt (goal : Goal) (proof prop : Expr) (generation : Nat) :

    Asserts a new fact prop with proof proof to the given goal.

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

      Asserts next fact in the goal fact queue.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        Equations
        Instances For
          partial def Lean.Meta.Grind.iterate.go (f : GoalGrindM (Option (List Goal))) (todo result : List Goal) :

          Asserts all facts in the goal fact queue.

          Equations
          Instances For