Documentation
Lean
.
Meta
.
Tactic
.
Simp
.
Diagnostics
Search
return to top
source
Imports
Lean.Meta.Diagnostics
Lean.Meta.Tactic.Simp.Types
Imported by
Lean
.
Meta
.
Simp
.
mkSimpDiagSummary
Lean
.
Meta
.
Simp
.
reportDiag
source
def
Lean
.
Meta
.
Simp
.
mkSimpDiagSummary
(counters :
PHashMap
Origin
Nat
)
(usedCounters? :
Option
(
PHashMap
Origin
Nat
)
:=
none
)
:
MetaM
DiagSummary
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
Simp
.
reportDiag
(diag :
Diagnostics
)
:
MetaM
Unit
Equations
One or more equations did not get rendered due to their size.
Instances For