diff --git a/src/Agda.hs b/src/Agda.hs index f44c4b8..26d70db 100644 --- a/src/Agda.hs +++ b/src/Agda.hs @@ -26,9 +26,7 @@ import Agda.Interaction.Base ( Command , CommandState(optionsOnReload) , IOTCM , initCommandState -#if MIN_VERSION_Agda(2,6,3) , parseIOTCM -#endif ) #if MIN_VERSION_Agda(2,6,4) import Agda.Syntax.Common.Pretty ( render, vcat ) @@ -180,14 +178,6 @@ handleCommandReq (CmdReq cmd) = do provideCommand iotcm return $ CmdRes Nothing -#if !MIN_VERSION_Agda(2,6,3) -parseIOTCM :: String -> Either String IOTCM -parseIOTCM raw = case listToMaybe $ reads raw of - Just (x, "" ) -> Right x - Just (_, remnent) -> Left $ "not consumed: " ++ remnent - _ -> Left $ "cannot read: " ++ raw -#endif - -------------------------------------------------------------------------------- getCommandLineOptions @@ -202,12 +192,8 @@ getCommandLineOptions = do result <- runExceptT $ do let p = parseBackendOptions builtinBackends merged defaultOptions -#if MIN_VERSION_Agda(2,6,3) let (r, _warns) = runOptM p (bs, opts) <- ExceptT $ pure r -#else - (bs, opts) <- ExceptT $ runOptM p -#endif return opts case result of -- something bad happened, use the default options instead diff --git a/src/Agda/Convert.hs b/src/Agda/Convert.hs index 190d034..de73acd 100644 --- a/src/Agda/Convert.hs +++ b/src/Agda/Convert.hs @@ -22,10 +22,7 @@ import Agda.Syntax.Concrete as C import Agda.Syntax.Internal (alwaysUnblock) import Agda.Syntax.Position (HasRange (getRange), Range, noRange) import Agda.Syntax.Scope.Base -import Agda.TypeChecking.Errors (getAllWarningsOfTCErr, prettyError) -#if MIN_VERSION_Agda(2,6,3) -import Agda.TypeChecking.Errors (explainWhyInScope) -#endif +import Agda.TypeChecking.Errors (getAllWarningsOfTCErr, prettyError, explainWhyInScope) import Agda.TypeChecking.Monad hiding (Function) import Agda.TypeChecking.Monad.MetaVars (withInteractionId) import Agda.TypeChecking.Pretty (prettyTCM) @@ -278,13 +275,8 @@ fromDisplayInfo = \case "Definitions about" <+> text (List.intercalate ", " $ words names) $$ nest 2 (align 10 hitDocs) return $ IR.DisplayInfoGeneric "Search About" [Unlabeled (Render.text $ show doc) Nothing Nothing] -#if MIN_VERSION_Agda(2,6,3) Info_WhyInScope why -> do doc <- explainWhyInScope why -#else - Info_WhyInScope s cwd v xs ms -> do - doc <- explainWhyInScope s cwd v xs ms -#endif return $ IR.DisplayInfoGeneric "Scope Info" [Unlabeled (Render.text $ show doc) Nothing Nothing] Info_Context ii ctx -> do doc <- localTCState (prettyResponseContexts ii False ctx) @@ -373,91 +365,6 @@ lispifyGoalSpecificDisplayInfo ii kind = localTCState $ -------------------------------------------------------------------------------- -#if !MIN_VERSION_Agda(2,6,3) -explainWhyInScope :: - String -> - FilePath -> - Maybe LocalVar -> - [AbstractName] -> - [AbstractModule] -> - TCM Doc -explainWhyInScope s _ Nothing [] [] = TCP.text (s ++ " is not in scope.") -explainWhyInScope s _ v xs ms = - TCP.vcat - [ TCP.text (s ++ " is in scope as"), - TCP.nest 2 $ TCP.vcat [variable v xs, modules ms] - ] - where - -- variable :: Maybe _ -> [_] -> TCM Doc - variable Nothing vs = names vs - variable (Just x) vs - | null vs = asVar - | otherwise = - TCP.vcat - [ TCP.sep [asVar, TCP.nest 2 $ shadowing x], - TCP.nest 2 $ names vs - ] - where - asVar :: TCM Doc - asVar = - "* a variable bound at" TCP.<+> TCP.prettyTCM (nameBindingSite $ localVar x) - shadowing :: LocalVar -> TCM Doc - shadowing (LocalVar _ _ []) = "shadowing" - shadowing _ = "in conflict with" - names = TCP.vcat . fmap pName - modules = TCP.vcat . fmap pMod - - pKind = \case - AxiomName -> "postulate" - ConName -> "constructor" - CoConName -> "coinductive constructor" - DataName -> "data type" - DisallowedGeneralizeName -> "generalizable variable from let open" - FldName -> "record field" - FunName -> "defined name" - GeneralizeName -> "generalizable variable" - MacroName -> "macro name" - PatternSynName -> "pattern synonym" - PrimName -> "primitive function" - QuotableName -> "quotable name" - -- previously DefName: - RecName -> "record type" - OtherDefName -> "defined name" - - pName :: AbstractName -> TCM Doc - pName a = - TCP.sep - [ "* a" - TCP.<+> pKind (anameKind a) - TCP.<+> TCP.text (prettyShow $ anameName a), - TCP.nest 2 "brought into scope by" - ] - TCP.$$ TCP.nest 2 (pWhy (nameBindingSite $ qnameName $ anameName a) (anameLineage a)) - pMod :: AbstractModule -> TCM Doc - pMod a = - TCP.sep - [ "* a module" TCP.<+> TCP.text (prettyShow $ amodName a), - TCP.nest 2 "brought into scope by" - ] - TCP.$$ TCP.nest 2 (pWhy (nameBindingSite $ qnameName $ mnameToQName $ amodName a) (amodLineage a)) - - pWhy :: Range -> WhyInScope -> TCM Doc - pWhy r Defined = "- its definition at" TCP.<+> TCP.prettyTCM r - pWhy r (Opened (C.QName x) w) | isNoName x = pWhy r w - pWhy r (Opened m w) = - "- the opening of" - TCP.<+> TCP.prettyTCM m - TCP.<+> "at" - TCP.<+> TCP.prettyTCM (getRange m) - TCP.$$ pWhy r w - pWhy r (Applied m w) = - "- the application of" - TCP.<+> TCP.prettyTCM m - TCP.<+> "at" - TCP.<+> TCP.prettyTCM (getRange m) - TCP.$$ pWhy r w -#endif - -- | Pretty-prints the context of the given meta-variable. prettyResponseContexts :: -- | Context of this meta-variable. diff --git a/src/Agda/Parser.hs b/src/Agda/Parser.hs index 2ab6897..5923248 100644 --- a/src/Agda/Parser.hs +++ b/src/Agda/Parser.hs @@ -7,9 +7,7 @@ module Agda.Parser where import Agda.Syntax.Parser (parseFile, runPMIO, tokensParser) import Agda.Syntax.Parser.Tokens (Token) import Agda.Syntax.Position (Position' (posPos), PositionWithoutFile, Range, getRange, rEnd', rStart') -#if MIN_VERSION_Agda(2,6,3) import Agda.Syntax.Position (RangeFile(RangeFile)) -#endif import Agda.Utils.FileName (mkAbsolute) import Monad ( ServerM ) import Control.Monad.State @@ -27,22 +25,12 @@ tokenAt :: LSP.Uri -> Text -> PositionWithoutFile -> ServerM (LspM Config) (Mayb tokenAt uri source position = case LSP.uriToFilePath uri of Nothing -> return Nothing Just filepath -> do - let file = -#if MIN_VERSION_Agda(2,6,3) - RangeFile (mkAbsolute filepath) Nothing -#else - mkAbsolute filepath -#endif + let file = RangeFile (mkAbsolute filepath) Nothing (result, _warnings) <- liftIO $ runPMIO $ do -- parse the file and get all tokens (r, _fileType) <- parseFile tokensParser file (unpack source) - let tokens = -#if MIN_VERSION_Agda(2,6,3) - fst r -#else - r -#endif + let tokens = fst r -- find the token at the position return $ find (pointedBy position) tokens case result of diff --git a/src/Agda/Position.hs b/src/Agda/Position.hs index 300602a..20a6cec 100644 --- a/src/Agda/Position.hs +++ b/src/Agda/Position.hs @@ -39,11 +39,7 @@ toAgdaRange table path (LSP.Range start end) = Range interval :: IntervalWithoutFile interval = Interval (toAgdaPositionWithoutFile table start) (toAgdaPositionWithoutFile table end) -#if MIN_VERSION_Agda(2,6,3) mkRangeFile path = RangeFile path Nothing -#else - mkRangeFile = id -#endif -- | LSP Position -> Agda PositionWithoutFile toAgdaPositionWithoutFile :: ToOffset -> LSP.Position -> PositionWithoutFile diff --git a/src/Render/Common.hs b/src/Render/Common.hs index 5e1579f..fbb5d63 100644 --- a/src/Render/Common.hs +++ b/src/Render/Common.hs @@ -17,7 +17,10 @@ import Agda.Syntax.Common QωOrigin(..), LensCohesion(getCohesion), NameId(..), - Erased(..), asQuantity, Lock(..), LockOrigin (..), + Erased(..), asQuantity, Lock(..), +#if MIN_VERSION_Agda(2,6,4) + LockOrigin (..), +#endif #if MIN_VERSION_Agda(2,7,0) OverlapMode (..), #endif @@ -38,11 +41,7 @@ instance Render NameId where -- | MetaId instance Render MetaId where -#if MIN_VERSION_Agda(2,6,3) render (MetaId n m) = text $ "_" ++ show n ++ "@" ++ show m -#else - render (MetaId n) = text $ "_" ++ show n -#endif -- | Relevance instance Render Relevance where @@ -112,8 +111,12 @@ renderQuantity a d = instance Render Lock where render = \case +#if MIN_VERSION_Agda(2,6,4) IsLock LockOLock -> "@lock" IsLock LockOTick -> "@tick" +#else + IsLock -> "@lock" +#endif IsNotLock -> mempty #if MIN_VERSION_Agda(2,7,0) diff --git a/src/Render/Concrete.hs b/src/Render/Concrete.hs index 5aa5f7e..e865ef2 100644 --- a/src/Render/Concrete.hs +++ b/src/Render/Concrete.hs @@ -120,10 +120,6 @@ instance Render Expr where Rec _ xs -> sep ["record", bracesAndSemicolons (fmap render xs)] RecUpdate _ e xs -> sep ["record" <+> render e, bracesAndSemicolons (fmap render xs)] -#if !MIN_VERSION_Agda(2,6,3) - ETel [] -> "()" - ETel tel -> fsep $ fmap render tel -#endif Quote _ -> "quote" QuoteTerm _ -> "quoteTerm" Unquote _ -> "unquote" @@ -550,10 +546,8 @@ instance Render Declaration where UnquoteDef _ xs t -> fsep ["unquoteDef" <+> fsep (fmap render xs) <+> "=", render t] Pragma pr -> sep ["{-#" <+> render pr, "#-}"] -#if MIN_VERSION_Agda(2,6,3) UnquoteData _ x xs e -> fsep [ hsep [ "unquoteData", render x, fsep (fmap render xs), "=" ], render e ] -#endif #if MIN_VERSION_Agda(2,6,4) Opaque _ ds -> namedBlock "opaque" ds @@ -697,10 +691,8 @@ instance Render Pragma where render (PolarityPragma _ q occs) = hsep ("POLARITY" : render q : fmap render occs) render (NoUniverseCheckPragma _) = "NO_UNIVERSE_CHECK" -#if MIN_VERSION_Agda(2,6,3) render (NotProjectionLikePragma _ q) = hsep [ "NOT_PROJECTION_LIKE", render q ] -#endif #if MIN_VERSION_Agda(2,7,0) render (InjectiveForInferencePragma _ i) = hsep $ ["INJECTIVE_FOR_INFERENCE", render i] @@ -716,20 +708,12 @@ instance Render Fixity where RightAssoc -> "infixr" NonAssoc -> "infix" -#if MIN_VERSION_Agda(2,6,3) instance Render NotationPart where render = \case IdPart x -> text $ rangedThing x HolePart{} -> "_" VarPart {} -> "_" WildPart{} -> "_" -#else -instance Render GenPart where - render (IdPart x) = text $ rangedThing x - render BindHole {} = "_" - render NormalHole {} = "_" - render WildHole {} = "_" -#endif instance Render Fixity' where render (Fixity' fix nota _) diff --git a/src/Render/Interaction.hs b/src/Render/Interaction.hs index e85dfa2..e352d57 100644 --- a/src/Render/Interaction.hs +++ b/src/Render/Interaction.hs @@ -109,10 +109,8 @@ instance (Render a, Render b) => Render (OutputConstraint a b) where "Check lock" <+> render lk <+> "allows" <+> render t render (UsableAtMod modality t) = "Is usable at" <+> render modality <+> render t -#if MIN_VERSION_Agda(2,6,3) render (DataSort _name expr) = fsep [ "Sort", render expr, "allows data/record definitions" ] -#endif -- | IPBoundary' instance Render c => Render (IPBoundary' c) where diff --git a/src/Render/Internal.hs b/src/Render/Internal.hs index 8caf8ca..2ef5994 100644 --- a/src/Render/Internal.hs +++ b/src/Render/Internal.hs @@ -25,12 +25,7 @@ instance Render a => Render (Substitution' a) where IdS -> "idS" EmptyS _ -> "emptyS" t :# rho -> mparens (p > 2) $ sep [pr 2 rho <> ",", renderPrec 3 t] -#if MIN_VERSION_Agda(2,6,3) - Strengthen _ _ rho -> -#else - Strengthen _ rho -> -#endif - mparens (p > 9) $ "strS" <+> pr 10 rho + Strengthen _ _ rho -> mparens (p > 9) $ "strS" <+> pr 10 rho Wk n rho -> mparens (p > 9) $ text ("wkS " ++ show n) <+> pr 10 rho Lift n rho -> mparens (p > 9) $ text ("liftS " ++ show n) <+> pr 10 rho @@ -170,9 +165,7 @@ instance Render Sort where MetaS x es -> renderPrec p $ MetaV x es DefS d es -> renderPrec p $ Def d es DummyS s -> parens $ text s -#if MIN_VERSION_Agda(2,6,3) IntervalUniv -> "IntervalUniv" -#endif #if MIN_VERSION_Agda(2,6,4) where suffix n = applyWhen (n /= 0) (++ show n) @@ -223,6 +216,4 @@ instance Render Blocker where render (UnblockOnAny us) = "any" <> parens (fsep $ punctuate "," $ map render $ Set.toList us) render (UnblockOnMeta m) = render m render (UnblockOnProblem pid) = "problem" <+> render pid -#if MIN_VERSION_Agda(2,6,3) render (UnblockOnDef q) = "definition" <+> render q -#endif diff --git a/src/Render/Position.hs b/src/Render/Position.hs index 7e11f92..c72c839 100644 --- a/src/Render/Position.hs +++ b/src/Render/Position.hs @@ -12,10 +12,8 @@ import Render.RichText instance Render AbsolutePath where render = text . filePath -#if MIN_VERSION_Agda(2,6,3) instance Render RangeFile where render = render . rangeFilePath -- TODO rangeFileName ? -#endif -------------------------------------------------------------------------------- diff --git a/src/Render/RichText.hs b/src/Render/RichText.hs index f195f8c..29a85de 100644 --- a/src/Render/RichText.hs +++ b/src/Render/RichText.hs @@ -214,10 +214,8 @@ instance {-# OVERLAPS #-} ToJSON Agda.SrcFile where instance ToJSON Agda.AbsolutePath where toJSON (Agda.AbsolutePath path) = toJSON path -#if MIN_VERSION_Agda(2,6,3) instance ToJSON Agda.RangeFile where toJSON (Agda.RangeFile path _maybeTopLevelModuleName) = toJSON path -#endif -------------------------------------------------------------------------------- diff --git a/src/Server/Handler.hs b/src/Server/Handler.hs index d73538a..845fd9b 100644 --- a/src/Server/Handler.hs +++ b/src/Server/Handler.hs @@ -100,12 +100,7 @@ inferTypeOfText filepath text = runCommandM $ do let norm = AsIs -- localStateCommandM: restore TC state afterwards, do we need this here? typ <- localStateCommandM $ do -#if MIN_VERSION_Agda(2,6,3) - (e, _attrs) -#else - e -#endif - <- lift $ runPM $ parse exprParser (unpack text) + (e, _attrs) <- lift $ runPM $ parse exprParser (unpack text) lift $ atTopLevel $ do concreteToAbstract_ e >>= typeInCurrent norm diff --git a/stack-9.2-Agda-2.6.2.2.yaml b/stack-9.2-Agda-2.6.2.2.yaml deleted file mode 100644 index 600fb65..0000000 --- a/stack-9.2-Agda-2.6.2.2.yaml +++ /dev/null @@ -1,21 +0,0 @@ -resolver: lts-20.26 -compiler: ghc-9.2.8 -# Allow a newer minor version of GHC than the snapshot specifies -compiler-check: newer-minor - -packages: -- . - -extra-deps: -- Agda-2.6.2.2 -- lsp-2.7.0.0@sha256:2a64b40a69fd9638056ca552d5660203019473061cff1d09dccc0c94e40a275c,3834 -- lsp-types-2.3.0.0@sha256:ca17a686bda5dc7ff04105ca7081dce5a90bcd050c8800a13efd68b7f0901f1c,34215 -- mod-0.2.0.1@sha256:eeb316fef3a8c12f4e83bbeeea748e74d75fca54d4498d574ace92e464adb05a,2409 -- row-types-1.0.1.2@sha256:4d4c7cb95d06a32b28ba977852d52a26b4c1f695ef083a6fd874ab6d79933b64,3071 - -flags: - agda-language-server: - Agda-2-6-2-2: true - Agda: - # optimise-heavily: true - enable-cluster-counting: true diff --git a/stack-9.2-Agda-2.6.2.2.yaml.lock b/stack-9.2-Agda-2.6.2.2.yaml.lock deleted file mode 100644 index e41f2ca..0000000 --- a/stack-9.2-Agda-2.6.2.2.yaml.lock +++ /dev/null @@ -1,47 +0,0 @@ -# This file was autogenerated by Stack. -# You should not edit this file by hand. -# For more information, please see the documentation at: -# https://docs.haskellstack.org/en/stable/lock_files - -packages: -- completed: - hackage: Agda-2.6.2.2@sha256:b69c2f317db2886cb387134af00a3e42a06fab6422686938797924d034255a55,37047 - pantry-tree: - sha256: 2f868d8f70a0f6bdbe96eff66ba1ec7a76b398cfc44dc57be525d7a67a44c9ab - size: 40002 - original: - hackage: Agda-2.6.2.2 -- completed: - hackage: lsp-2.7.0.0@sha256:2a64b40a69fd9638056ca552d5660203019473061cff1d09dccc0c94e40a275c,3834 - pantry-tree: - sha256: 630a5e18d7783c35a296268959c8d9348ee6dc94540047ea58146b310d8de941 - size: 1120 - original: - hackage: lsp-2.7.0.0@sha256:2a64b40a69fd9638056ca552d5660203019473061cff1d09dccc0c94e40a275c,3834 -- completed: - hackage: lsp-types-2.3.0.0@sha256:ca17a686bda5dc7ff04105ca7081dce5a90bcd050c8800a13efd68b7f0901f1c,34215 - pantry-tree: - sha256: 0bf22e394dc804c8cee74d19a7f38021cfd48a15082b39a14753c037f2a64288 - size: 51996 - original: - hackage: lsp-types-2.3.0.0@sha256:ca17a686bda5dc7ff04105ca7081dce5a90bcd050c8800a13efd68b7f0901f1c,34215 -- completed: - hackage: mod-0.2.0.1@sha256:eeb316fef3a8c12f4e83bbeeea748e74d75fca54d4498d574ace92e464adb05a,2409 - pantry-tree: - sha256: d469d7e415c1593f052d3ca647e4085ab759be378d25ca7d2eea0aab0083ce38 - size: 590 - original: - hackage: mod-0.2.0.1@sha256:eeb316fef3a8c12f4e83bbeeea748e74d75fca54d4498d574ace92e464adb05a,2409 -- completed: - hackage: row-types-1.0.1.2@sha256:4d4c7cb95d06a32b28ba977852d52a26b4c1f695ef083a6fd874ab6d79933b64,3071 - pantry-tree: - sha256: 6a3617038d3970095100d14d026c396002a115700500cf3004ffb67ae5a75611 - size: 1060 - original: - hackage: row-types-1.0.1.2@sha256:4d4c7cb95d06a32b28ba977852d52a26b4c1f695ef083a6fd874ab6d79933b64,3071 -snapshots: -- completed: - sha256: 5a59b2a405b3aba3c00188453be172b85893cab8ebc352b1ef58b0eae5d248a2 - size: 650475 - url: https://raw.githubusercontent.com/commercialhaskell/stackage-snapshots/master/lts/20/26.yaml - original: lts-20.26 diff --git a/stack-9.2-Agda-2.6.4.3.yaml.lock b/stack-9.2-Agda-2.6.4.3.yaml.lock index 4e8b7e4..37f50db 100644 --- a/stack-9.2-Agda-2.6.4.3.yaml.lock +++ b/stack-9.2-Agda-2.6.4.3.yaml.lock @@ -25,6 +25,13 @@ packages: size: 51996 original: hackage: lsp-types-2.3.0.0@sha256:ca17a686bda5dc7ff04105ca7081dce5a90bcd050c8800a13efd68b7f0901f1c,34215 +- completed: + hackage: lsp-test-0.17.1.0@sha256:f54757a564b46783cf67b13f4cb4ebc45e43f5afc3604d9757ee387c091b73e9,4406 + pantry-tree: + sha256: 66797a8efd50812189c410310dc0a9b72858ea3a3e78764e9cedd8f406df2564 + size: 1561 + original: + hackage: lsp-test-0.17.1.0@sha256:f54757a564b46783cf67b13f4cb4ebc45e43f5afc3604d9757ee387c091b73e9,4406 - completed: hackage: mod-0.2.0.1@sha256:eeb316fef3a8c12f4e83bbeeea748e74d75fca54d4498d574ace92e464adb05a,2409 pantry-tree: diff --git a/stack-9.2-Agda-2.6.4.yaml b/stack-9.2-Agda-2.6.4.yaml deleted file mode 100644 index 52cd6b1..0000000 --- a/stack-9.2-Agda-2.6.4.yaml +++ /dev/null @@ -1,18 +0,0 @@ -resolver: lts-20.26 -compiler: ghc-9.2.8 -# Allow a newer minor version of GHC than the snapshot specifies -compiler-check: newer-minor - -packages: -- . - -extra-deps: -- Agda-2.6.4 -- lsp-2.7.0.0@sha256:2a64b40a69fd9638056ca552d5660203019473061cff1d09dccc0c94e40a275c,3834 -- lsp-types-2.3.0.0@sha256:ca17a686bda5dc7ff04105ca7081dce5a90bcd050c8800a13efd68b7f0901f1c,34215 -- mod-0.2.0.1@sha256:eeb316fef3a8c12f4e83bbeeea748e74d75fca54d4498d574ace92e464adb05a,2409 -- row-types-1.0.1.2@sha256:4d4c7cb95d06a32b28ba977852d52a26b4c1f695ef083a6fd874ab6d79933b64,3071 -flags: - Agda: - # optimise-heavily: true - enable-cluster-counting: true diff --git a/stack-9.2-Agda-2.6.4.yaml.lock b/stack-9.2-Agda-2.6.4.yaml.lock deleted file mode 100644 index 986bbcc..0000000 --- a/stack-9.2-Agda-2.6.4.yaml.lock +++ /dev/null @@ -1,47 +0,0 @@ -# This file was autogenerated by Stack. -# You should not edit this file by hand. -# For more information, please see the documentation at: -# https://docs.haskellstack.org/en/stable/lock_files - -packages: -- completed: - hackage: Agda-2.6.4@sha256:298bc3b261ad034bf4ee788834a4d296aa5c2f6ea17ac4bef44e3daea53a7cd8,28443 - pantry-tree: - sha256: 6c811b2ff8aa666ba301666e87d9234993d841dd370d47f8398379cd943e47bb - size: 42645 - original: - hackage: Agda-2.6.4 -- completed: - hackage: lsp-2.7.0.0@sha256:2a64b40a69fd9638056ca552d5660203019473061cff1d09dccc0c94e40a275c,3834 - pantry-tree: - sha256: 630a5e18d7783c35a296268959c8d9348ee6dc94540047ea58146b310d8de941 - size: 1120 - original: - hackage: lsp-2.7.0.0@sha256:2a64b40a69fd9638056ca552d5660203019473061cff1d09dccc0c94e40a275c,3834 -- completed: - hackage: lsp-types-2.3.0.0@sha256:ca17a686bda5dc7ff04105ca7081dce5a90bcd050c8800a13efd68b7f0901f1c,34215 - pantry-tree: - sha256: 0bf22e394dc804c8cee74d19a7f38021cfd48a15082b39a14753c037f2a64288 - size: 51996 - original: - hackage: lsp-types-2.3.0.0@sha256:ca17a686bda5dc7ff04105ca7081dce5a90bcd050c8800a13efd68b7f0901f1c,34215 -- completed: - hackage: mod-0.2.0.1@sha256:eeb316fef3a8c12f4e83bbeeea748e74d75fca54d4498d574ace92e464adb05a,2409 - pantry-tree: - sha256: d469d7e415c1593f052d3ca647e4085ab759be378d25ca7d2eea0aab0083ce38 - size: 590 - original: - hackage: mod-0.2.0.1@sha256:eeb316fef3a8c12f4e83bbeeea748e74d75fca54d4498d574ace92e464adb05a,2409 -- completed: - hackage: row-types-1.0.1.2@sha256:4d4c7cb95d06a32b28ba977852d52a26b4c1f695ef083a6fd874ab6d79933b64,3071 - pantry-tree: - sha256: 6a3617038d3970095100d14d026c396002a115700500cf3004ffb67ae5a75611 - size: 1060 - original: - hackage: row-types-1.0.1.2@sha256:4d4c7cb95d06a32b28ba977852d52a26b4c1f695ef083a6fd874ab6d79933b64,3071 -snapshots: -- completed: - sha256: 5a59b2a405b3aba3c00188453be172b85893cab8ebc352b1ef58b0eae5d248a2 - size: 650475 - url: https://raw.githubusercontent.com/commercialhaskell/stackage-snapshots/master/lts/20/26.yaml - original: lts-20.26