Documentation

Lean.Meta.Diagnostics

def Lean.Meta.collectAboveThreshold {α : Type u_1} [BEq α] [Hashable α] (counters : PHashMap α Nat) (threshold : Nat) (p : αBool) (lt : ααBool) :
Array (α × Nat)
Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def Lean.Meta.subCounters {α : Type u_1} [BEq α] [Hashable α] (newCounters oldCounters : PHashMap α Nat) :
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      Instances For
        Equations
        • s.isEmpty = s.data.isEmpty
        Instances For
          def Lean.Meta.mkDiagSummary (cls : Name) (counters : PHashMap Name Nat) (p : NameBool := fun (x : Name) => true) :
          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
                Equations
                Instances For
                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    def Lean.Meta.appendSection (m : MessageData) (cls : Name) (header : String) (s : DiagSummary) (resultSummary : Bool := true) :

                    We use below that this returns m unchanged if s.isEmpty

                    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