File tree 4 files changed +7
-7
lines changed
4 files changed +7
-7
lines changed Original file line number Diff line number Diff line change @@ -140,7 +140,7 @@ compileFun' withSig def@Defn{..} = do
140
140
-- We only instantiate the clauses to the current module parameters
141
141
-- if the current module isn't the toplevel module
142
142
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
144
144
let clauses = if weAreOnTop then filtered else filtered `apply` pars
145
145
146
146
typ <- if weAreOnTop then pure defType else piApplyM defType pars
@@ -228,7 +228,7 @@ compileClause' curModule projName x ty c@Clause{..} = do
228
228
compilePats :: Type -> NAPs -> C [Hs. Pat () ]
229
229
compilePats _ [] = pure []
230
230
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)
232
232
unlessM (asks copatternsEnabled `or2M` (isJust <$> isUnboxProjection pn)) $
233
233
genericDocError =<< " not supported in Haskell: copatterns"
234
234
@@ -239,7 +239,7 @@ compilePats ty ((namedArg -> ProjP po pn):ps) = do
239
239
240
240
compilePats ty ((namedArg -> pat): ps) = do
241
241
(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
243
243
let rest = compilePats (absApp b (patternToTerm pat)) ps
244
244
compileDom a >>= \ case
245
245
DOInstance -> rest
Original file line number Diff line number Diff line change @@ -128,7 +128,7 @@ primWord64FromNat ty args = compileArgs ty args >>= \case
128
128
-- should really be named compileVar, TODO: rename compileVar
129
129
compileVar :: Int -> Type -> [Term ] -> C (Hs. Exp () )
130
130
compileVar i ty es = do
131
- reportSDoc " agda2hs.compile.term" 10 $ text " Reached variable"
131
+ reportSDoc " agda2hs.compile.term" 15 $ text " Reached variable"
132
132
name <- compileDBVar i
133
133
compileApp (hsVar name) ty es
134
134
@@ -383,7 +383,7 @@ compileCon h i ty args = do
383
383
compileTerm :: Type -> Term -> C (Hs. Exp () )
384
384
compileTerm ty v = do
385
385
386
- reportSDoc " agda2hs.compile" 7 $ text " compiling term:" <+> prettyTCM v
386
+ reportSDoc " agda2hs.compile.term " 10 $ text " compiling term:" <+> prettyTCM v
387
387
388
388
let bad s t = genericDocError =<< vcat
389
389
[ text " agda2hs: cannot compile" <+> text (s ++ " :" )
Original file line number Diff line number Diff line change @@ -91,7 +91,7 @@ compileTopLevelType
91
91
-> (Hs. Type () -> C a ) -- ^ Continuation with the compiled type.
92
92
-> C a
93
93
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
95
95
-- NOTE(flupe): even though we only quantify variable for definitions inside anonymous modules,
96
96
-- they will still get quantified over the toplevel module parameters.
97
97
weAreOnTop <- isJust <$> liftTCM (currentModule >>= isTopLevelModule)
Original file line number Diff line number Diff line change @@ -238,7 +238,7 @@ isInlinedFunction q = do
238
238
239
239
checkInstance :: Term -> C ()
240
240
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
242
242
t <- infer u
243
243
reportSDoc " agda2hs.checkInstance" 15 $ text " inferred type:" <+> prettyTCM t
244
244
(m, v) <- newInstanceMeta " " t
You can’t perform that action at this time.
0 commit comments