Documentation

Lean.Meta.Tactic.Grind.Core

Tries to apply beta-reductiong using the parent applications of the functions in fns with the lambda expressions in lams.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def Lean.Meta.Grind.addNewEq (lhs rhs proof : Expr) (generation : Nat) :

    Internalizes lhs and rhs, and then adds equality lhs = rhs.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      def Lean.Meta.Grind.add (fact proof : Expr) (generation : Nat := 0) :

      Adds a new fact justified by the given proof and using the given generation.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        def Lean.Meta.Grind.add.go (proof : Expr) (generation : Nat := 0) (p : Expr) (isNeg : Bool) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          def Lean.Meta.Grind.add.goFact (proof : Expr) (generation : Nat := 0) (p : Expr) (isNeg : Bool) :
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            def Lean.Meta.Grind.add.goEq (proof : Expr) (generation : Nat := 0) (p lhs rhs : Expr) (isNeg isHEq : Bool) :
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def Lean.Meta.Grind.addHypothesis (fvarId : FVarId) (generation : Nat := 0) :

              Adds a new hypothesis.

              Equations
              Instances For