Documentation

Lean.Elab.Tactic.Conv.Congr

def Lean.Elab.Tactic.Conv.congr (mvarId : Lean.MVarId) (addImplicitArgs : Bool := false) (nameSubgoals : Bool := true) :
Instances For
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      Implementation of arg 0.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        def Lean.Elab.Tactic.Conv.congrArgForall (tacticName : String) (domain : Bool) (mvarId : Lean.MVarId) (lhs rhs : Lean.Expr) :

        Implements arg for foralls. If domain is true, accesses the domain, otherwise accesses the codomain.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          def Lean.Elab.Tactic.Conv.congrArgN (tacticName : String) (mvarId : Lean.MVarId) (i : Int) (explicit : Bool) :

          Implementation of arg i.

          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
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For