Skip to content

Commit 3ab718a

Browse files
committed
Update a few debug levels
1 parent bb65f8a commit 3ab718a

File tree

4 files changed

+7
-7
lines changed

4 files changed

+7
-7
lines changed

src/Agda2Hs/Compile/Function.hs

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -140,7 +140,7 @@ compileFun' withSig def@Defn{..} = do
140140
-- We only instantiate the clauses to the current module parameters
141141
-- if the current module isn't the toplevel module
142142
unless weAreOnTop $
143-
reportSDoc "agda2hs.compile.type" 6 $ "Applying module parameters to clauses: " <+> prettyTCM pars
143+
reportSDoc "agda2hs.compile.type" 8 $ "Applying module parameters to clauses: " <+> prettyTCM pars
144144
let clauses = if weAreOnTop then filtered else filtered `apply` pars
145145

146146
typ <- if weAreOnTop then pure defType else piApplyM defType pars
@@ -228,7 +228,7 @@ compileClause' curModule projName x ty c@Clause{..} = do
228228
compilePats :: Type -> NAPs -> C [Hs.Pat ()]
229229
compilePats _ [] = pure []
230230
compilePats ty ((namedArg -> ProjP po pn):ps) = do
231-
reportSDoc "agda2hs.compile" 6 $ "compiling copattern: " <+> text (prettyShow pn)
231+
reportSDoc "agda2hs.compile" 10 $ "compiling copattern: " <+> text (prettyShow pn)
232232
unlessM (asks copatternsEnabled `or2M` (isJust <$> isUnboxProjection pn)) $
233233
genericDocError =<< "not supported in Haskell: copatterns"
234234

@@ -239,7 +239,7 @@ compilePats ty ((namedArg -> ProjP po pn):ps) = do
239239

240240
compilePats ty ((namedArg -> pat):ps) = do
241241
(a, b) <- mustBePi ty
242-
reportSDoc "agda2hs.compile.pattern" 5 $ text "Compiling pattern:" <+> prettyTCM pat
242+
reportSDoc "agda2hs.compile.pattern" 10 $ text "Compiling pattern:" <+> prettyTCM pat
243243
let rest = compilePats (absApp b (patternToTerm pat)) ps
244244
compileDom a >>= \case
245245
DOInstance -> rest

src/Agda2Hs/Compile/Term.hs

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -128,7 +128,7 @@ primWord64FromNat ty args = compileArgs ty args >>= \case
128128
-- should really be named compileVar, TODO: rename compileVar
129129
compileVar :: Int -> Type -> [Term] -> C (Hs.Exp ())
130130
compileVar i ty es = do
131-
reportSDoc "agda2hs.compile.term" 10 $ text "Reached variable"
131+
reportSDoc "agda2hs.compile.term" 15 $ text "Reached variable"
132132
name <- compileDBVar i
133133
compileApp (hsVar name) ty es
134134

@@ -383,7 +383,7 @@ compileCon h i ty args = do
383383
compileTerm :: Type -> Term -> C (Hs.Exp ())
384384
compileTerm ty v = do
385385

386-
reportSDoc "agda2hs.compile" 7 $ text "compiling term:" <+> prettyTCM v
386+
reportSDoc "agda2hs.compile.term" 10 $ text "compiling term:" <+> prettyTCM v
387387

388388
let bad s t = genericDocError =<< vcat
389389
[ text "agda2hs: cannot compile" <+> text (s ++ ":")

src/Agda2Hs/Compile/Type.hs

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -91,7 +91,7 @@ compileTopLevelType
9191
-> (Hs.Type () -> C a) -- ^ Continuation with the compiled type.
9292
-> C a
9393
compileTopLevelType keepType t cont = do
94-
reportSDoc "agda2hs.compile.type" 12 $ text "Compiling top-level type" <+> prettyTCM t
94+
reportSDoc "agda2hs.compile.type" 8 $ text "Compiling top-level type" <+> prettyTCM t
9595
-- NOTE(flupe): even though we only quantify variable for definitions inside anonymous modules,
9696
-- they will still get quantified over the toplevel module parameters.
9797
weAreOnTop <- isJust <$> liftTCM (currentModule >>= isTopLevelModule)

src/Agda2Hs/Compile/Utils.hs

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -238,7 +238,7 @@ isInlinedFunction q = do
238238

239239
checkInstance :: Term -> C ()
240240
checkInstance u | varOrDef u = liftTCM $ noConstraints $ do
241-
reportSDoc "agda2hs.checkInstance" 5 $ text "checkInstance" <+> prettyTCM u
241+
reportSDoc "agda2hs.checkInstance" 12 $ text "checkInstance" <+> prettyTCM u
242242
t <- infer u
243243
reportSDoc "agda2hs.checkInstance" 15 $ text " inferred type:" <+> prettyTCM t
244244
(m, v) <- newInstanceMeta "" t

0 commit comments

Comments
 (0)