Skip to content

Commit

Permalink
Whitespace
Browse files Browse the repository at this point in the history
  • Loading branch information
jespercockx committed Jul 23, 2024
1 parent 593f55d commit 4fa1990
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 5 deletions.
2 changes: 1 addition & 1 deletion src/Agda2Hs/Compile/Record.hs
Original file line number Diff line number Diff line change
Expand Up @@ -177,7 +177,7 @@ checkUnboxPragma def = do
-- recRecursive can be used again after agda 2.6.4.2 is released
-- see agda/agda#7042
unless (all null recMutual) $ genericDocError
=<< text "Unboxed record" <+> prettyTCM (defName def)
=<< text "Unboxed record" <+> prettyTCM (defName def)
<+> text "cannot be recursive"

TelV tel _ <- telViewUpTo recPars (defType def)
Expand Down
8 changes: 4 additions & 4 deletions src/Agda2Hs/Compile/Type.hs
Original file line number Diff line number Diff line change
Expand Up @@ -129,7 +129,7 @@ compileType t = do
-- TODO: we should also drop lambdas that can be erased based on their type
-- (e.g. argument is of type Level/Size or in a Prop) but currently we do
-- not have access to the type of the lambda here.
Lam argInfo restAbs
Lam argInfo restAbs
| hasQuantity0 argInfo -> underAbstraction_ restAbs compileType
| otherwise -> genericDocError =<< text "Not supported: type-level lambda" <+> prettyTCM t

Expand All @@ -144,7 +144,7 @@ compileTypeArgs ty (x:xs) = do
reportSDoc "agda2hs.compile.type" 16 $ text "compileTypeArgs x =" <+> prettyTCM x
reportSDoc "agda2hs.compile.type" 16 $ text " a =" <+> prettyTCM a
reportSDoc "agda2hs.compile.type" 16 $ text " modality =" <+> prettyTCM (getModality a)
let rest = compileTypeArgs (absApp b $ unArg x) xs
let rest = compileTypeArgs (absApp b $ unArg x) xs
let fail msg = genericDocError =<< (text msg <> text ":") <+> parens (prettyTCM (absName b) <+> text ":" <+> prettyTCM (unDom a))
compileDom a >>= \case
DODropped -> rest
Expand Down Expand Up @@ -217,7 +217,7 @@ compileDom a = do
isErasable <- pure (not $ usableModality a) `or2M` canErase (unDom a)
isClassConstraint <- pure (isInstance a) `and2M` isClassType (unDom a)
isType <- endsInSort (unDom a)
return $ if
return $ if
| isErasable -> DODropped
| isClassConstraint -> DOInstance
| isType -> DOType
Expand All @@ -240,7 +240,7 @@ compileDomType x a =
-- come from a module parameter.
ctx <- getContextSize
npars <- size <$> (lookupSection =<< currentModule)
if ctx < npars
if ctx < npars
then do
tellExtension Hs.ScopedTypeVariables
return $ DomForall $ Hs.UnkindedVar () $ Hs.Ident () x
Expand Down

0 comments on commit 4fa1990

Please sign in to comment.