@[export lean_get_profiler_threshold]
Instances For
@[extern lean_profileit]
def
Lean.profileit
{α : Type}
(category : String)
(opts : Lean.Options)
(fn : Unit → α)
(decl : Lean.Name := Lean.Name.anonymous)
:
α
Print and accumulate run time of act
when option profiler
is set to true
.
Equations
- Lean.profileit category opts fn decl = fn ()
Instances For
unsafe def
Lean.profileitIOUnsafe
{ε α : Type}
(category : String)
(opts : Lean.Options)
(act : EIO ε α)
(decl : Lean.Name := Lean.Name.anonymous)
:
EIO ε α
Instances For
@[implemented_by Lean.profileitIOUnsafe]
def
Lean.profileitIO
{ε α : Type}
(category : String)
(opts : Lean.Options)
(act : EIO ε α)
(decl : Lean.Name := Lean.Name.anonymous)
:
EIO ε α
Instances For
def
Lean.profileitM
{m : Type → Type}
(ε : Type)
[MonadFunctorT (EIO ε) m]
{α : Type}
(category : String)
(opts : Lean.Options)
(act : m α)
(decl : Lean.Name := Lean.Name.anonymous)
:
m α