Agda-2.2.10: A dependently typed functional programming language and proof assistant
Source code
Contents
Index
Agda.TypeChecking.Monad.Trace
Contents
Trace
Synopsis
interestingCall
::
Closure
Call
->
Bool
traceCall
::
MonadTCM
tcm => (
Maybe
r ->
Call
) -> tcm a -> tcm a
traceCall_
::
MonadTCM
tcm => (
Maybe
()
->
Call
) -> tcm r -> tcm r
traceCallCPS
::
MonadTCM
tcm => (
Maybe
r ->
Call
) -> (r -> tcm a) -> ((r -> tcm a) -> tcm b) -> tcm b
traceCallCPS_
::
MonadTCM
tcm => (
Maybe
()
->
Call
) -> tcm a -> (tcm a -> tcm b) -> tcm b
getCurrentRange
::
MonadTCM
tcm => tcm
Range
setCurrentRange
::
MonadTCM
tcm =>
Range
-> tcm a -> tcm a
Trace
interestingCall
::
Closure
Call
->
Bool
Source
traceCall
::
MonadTCM
tcm => (
Maybe
r ->
Call
) -> tcm a -> tcm a
Source
Record a function call in the trace.
traceCall_
::
MonadTCM
tcm => (
Maybe
()
->
Call
) -> tcm r -> tcm r
Source
traceCallCPS
::
MonadTCM
tcm => (
Maybe
r ->
Call
) -> (r -> tcm a) -> ((r -> tcm a) -> tcm b) -> tcm b
Source
traceCallCPS_
::
MonadTCM
tcm => (
Maybe
()
->
Call
) -> tcm a -> (tcm a -> tcm b) -> tcm b
Source
getCurrentRange
::
MonadTCM
tcm => tcm
Range
Source
setCurrentRange
::
MonadTCM
tcm =>
Range
-> tcm a -> tcm a
Source
Produced by
Haddock
version 2.6.1