Documentation

Lean.Meta.Tactic.Grind.ForallProp

If parent is a projection-application proj_i c, check whether the root of the equivalence class containing c is a constructor-application ctor ... a_i .... If so, internalize the term proj_i (ctor ... a_i ...) and add the equality proj_i (ctor ... a_i ...) = a_i.

Equations
Instances For

    Given a proof of an EMatchTheorem, returns true, if there are no anchor references restricting the search, or there is an anchor references ref s.t. ref matches proof.

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

          Applies the following rewriting rules:

          • Grind.imp_true_eq
          • Grind.imp_false_eq
          • Grind.forall_imp_eq_or
          • Grind.true_imp_eq
          • Grind.false_imp_eq
          • Grind.imp_self_eq
          • forall_true
          • forall_false
          • Grind.forall_or_forall
          • Grind.forall_forall_or
          • Grind.forall_and
          Equations
          Instances For

            Applies the following rewriting rules:

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