Skip to content

Commit

Permalink
[ agda#6055, 2.6.3 final ] Agda.cabal and stack-XYZ.yaml files.
Browse files Browse the repository at this point in the history
    * Removed Cabal test-suite
    * Removed -Werror
    * Cleaning stack-XYZ.yaml files
      + Removed QuickCheck dependency
      + Removed tasty-* dependencies
      + Removed package section

[ci skip]
  • Loading branch information
asr authored and JobPetrovcic committed Apr 5, 2024
1 parent 8f98e77 commit 55b1c54
Show file tree
Hide file tree
Showing 8 changed files with 0 additions and 317 deletions.
276 changes: 0 additions & 276 deletions Agda.cabal
Original file line number Diff line number Diff line change
Expand Up @@ -854,7 +854,6 @@ library
ghc-options: -fprint-potential-instances
-- Initially, we disable all the warnings.
-w
-Werror
-- This option must be the first one after disabling the
-- warnings. See Issue #2094.
-Wunrecognised-warning-flags
Expand Down Expand Up @@ -891,7 +890,6 @@ library
else
ghc-options: -fprint-potential-instances
-- ASR (2022-05-31). Workaround to Issue #5932.
-Werror
-Werror=unrecognised-warning-flags
-Werror=deprecated-flags
-Werror=deriving-typeable
Expand Down Expand Up @@ -1026,277 +1024,3 @@ executable agda-mode
, filepath >= 1.4.1.0 && < 1.5
, process >= 1.4.2.0 && < 1.7
default-language: Haskell2010

-- Cabal testsuite integration has some serious bugs, but we
-- can still make it work. See also:
-- https://github.com/haskell/cabal/issues/1938
-- https://github.com/haskell/cabal/issues/2214
-- https://github.com/haskell/cabal/issues/1953
--
-- This test suite should only be run using the Makefile.
-- The Makefile sets up the required environment,
-- executing the tests using cabal directly is almost
-- guaranteed to fail. See also Issue 1490.
test-suite agda-tests
type: exitcode-stdio-1.0
hs-source-dirs: test/
main-is: Main.hs
other-modules: Bugs.Tests
, Compiler.Tests
, CubicalSucceed.Tests
, Fail.Tests
, Interactive.Tests
, Internal.Compiler.MAlonzo.Encode
, Internal.Helpers
, Internal.Interaction.Highlighting.Precise
, Internal.Interaction.Highlighting.Range
, Internal.Interaction.Library
, Internal.Interaction.Options
, Internal.Syntax.Abstract.Name
, Internal.Syntax.Common
, Internal.Syntax.Concrete.Name
, Internal.Syntax.Internal
, Internal.Syntax.Parser.Parser
, Internal.Syntax.Position
, Internal.Termination.CallGraph
, Internal.Termination.CallMatrix
, Internal.Termination.Order
, Internal.Termination.Semiring
, Internal.Termination.SparseMatrix
, Internal.Termination.Termination
, Internal.Tests
, Internal.TypeChecking
, Internal.TypeChecking.Free
, Internal.TypeChecking.Free.Lazy
, Internal.TypeChecking.Generators
, Internal.TypeChecking.Irrelevance
, Internal.TypeChecking.Monad.Base
, Internal.TypeChecking.Positivity
, Internal.TypeChecking.Positivity.Occurrence
, Internal.TypeChecking.Rules.LHS.Problem
, Internal.TypeChecking.SizedTypes
, Internal.TypeChecking.SizedTypes.Syntax
, Internal.TypeChecking.SizedTypes.WarshallSolver
, Internal.TypeChecking.Substitute
, Internal.Utils.AssocList
, Internal.Utils.Bag
, Internal.Utils.BiMap
, Internal.Utils.Cluster
, Internal.Utils.Either
, Internal.Utils.Favorites
, Internal.Utils.FileName
, Internal.Utils.Graph.AdjacencyMap.Unidirectional
, Internal.Utils.IntSet
, Internal.Utils.List
, Internal.Utils.List1
, Internal.Utils.List2
, Internal.Utils.ListT
, Internal.Utils.Maybe.Strict
, Internal.Utils.Monoid
, Internal.Utils.PartialOrd
, Internal.Utils.Permutation
, Internal.Utils.RangeMap
, Internal.Utils.SmallSet
, Internal.Utils.Three
, Internal.Utils.Trie
, Internal.Utils.Warshall
, LaTeXAndHTML.Tests
, LibSucceed.Tests
, Succeed.Tests
, UserManual.Tests
, Utils

-- Andreas, 2021-08-26, see https://github.com/haskell/cabal/issues/7577
-- Since 'agda-tests' wants to call 'agda', we have to add it here,
-- should we want to run 'cabal test'.
build-tool-depends: Agda:agda

build-depends: Agda
, array
, base
, bytestring
, containers
, directory
, filepath
, filemanip >= 0.3.6.3 && < 0.4
, mtl
, process
, process-extras >= 0.3.0 && < 0.3.4 || >= 0.4.1.3 && < 0.5 || >= 0.7.1 && < 0.8
, QuickCheck >= 2.14.1 && < 2.15
, regex-tdfa
, split
, strict
, tasty >= 1.1.0.4 && < 1.5
, tasty-hunit >= 0.9.2 && < 0.11
, tasty-quickcheck >= 0.9.2 && < 0.11
-- tasty-silver 3.1.13 has option --ansi-tricks=false
-- NB: tasty-silver 3.2 requires tasty >= 1.4
-- tasty-silver < 3.3 does not work interactively under Windows
, tasty-silver >= 3.1.13 && < 3.4
, temporary >= 1.2.0.3 && < 1.4
, text
, unix-compat >= 0.4.3.1 && < 0.7
, unordered-containers
, uri-encode

-- Andreas (2021-10-11): tasty-silver < 3.3 does not work interactively under Windows
if os(windows)
build-depends: tasty-silver >= 3.3

default-language: Haskell2010

-- NOTE: If adding or removing default extensions, also change:
-- .hlint.yaml
-- This should also use the same extensions as the `library` target above.
default-extensions: BangPatterns
, ConstraintKinds
--L-T Chen (2019-07-15):
-- Enabling DataKinds only locally makes the compile time
-- slightly shorter, see PR #3920.
--, DataKinds
, DefaultSignatures
, DeriveDataTypeable
, DeriveFoldable
, DeriveFunctor
, DeriveGeneric
, DeriveTraversable
, ExistentialQuantification
, FlexibleContexts
, FlexibleInstances
, FunctionalDependencies
, GeneralizedNewtypeDeriving
, InstanceSigs
, LambdaCase
, MultiParamTypeClasses
, MultiWayIf
, NamedFieldPuns
, OverloadedStrings
, PatternSynonyms
, RankNTypes
, RecordWildCards
, ScopedTypeVariables
, StandaloneDeriving
, TupleSections
, TypeFamilies
, TypeOperators
, TypeSynonymInstances

if flag(optimise-heavily)
ghc-options: -fexpose-all-unfoldings
-fspecialise-aggressively

if impl(ghc <= 8.0.2)
ghc-options: -threaded
-- Initially, we disable all the warnings.
-w
-Werror
-- This option must be the first one after disabling the
-- warnings. See Issue #2094.
-Wunrecognised-warning-flags
-Wdeprecated-flags
-Wderiving-typeable
-Wdodgy-exports
-Wdodgy-foreign-imports
-Wdodgy-imports
-Wduplicate-exports
-Wempty-enumerations
-Widentities
-- #6137: GHC 8.0 has no COMPLETE pragma, so we have to turn off the completeness checker
-- -Wincomplete-patterns
-- -Wincomplete-record-updates
-Winline-rule-shadowing
-Wmissing-fields
-Wmissing-methods
-Wmissing-pattern-synonym-signatures
-Wmissing-signatures
-Wnoncanonical-monad-instances
-Wnoncanonical-monoid-instances
-Woverflowed-literals
-- #6137: GHC 8.0 has no COMPLETE pragma, so we have to turn off the completeness checker
-- -Woverlapping-patterns
-Wsemigroup
-Wtabs
-Wtyped-holes
-Wunrecognised-pragmas
-Wunticked-promoted-constructors
-Wunused-do-bind
-Wunused-foralls
-Wwarnings-deprecations
-Wwrong-do-bind
else
ghc-options: -threaded
-- ASR (2022-05-31). Workaround to Issue #5932.
-Werror
-Werror=unrecognised-warning-flags
-Werror=deprecated-flags
-Werror=deriving-typeable
-Werror=dodgy-exports
-Werror=dodgy-foreign-imports
-Werror=dodgy-imports
-Werror=duplicate-exports
-Werror=empty-enumerations
-Werror=identities
-Werror=inline-rule-shadowing
-Werror=missing-fields
-Werror=missing-methods
-Werror=missing-pattern-synonym-signatures
-Werror=missing-signatures
-Werror=noncanonical-monad-instances
-Werror=noncanonical-monoid-instances
-Werror=overflowed-literals
-Werror=overlapping-patterns
-Werror=semigroup
-Werror=tabs
-Werror=typed-holes
-Werror=unrecognised-pragmas
-Werror=unticked-promoted-constructors
-Werror=unused-do-bind
-Werror=unused-foralls
-Werror=warnings-deprecations
-Werror=wrong-do-bind

-- ASR (2017-04-11). TODO: Using -Werror=missing-home-modules generates an
-- error.
if impl(ghc >= 8.2)
ghc-options: -Werror=cpp-undef
-Werror=simplifiable-class-constraints
-Werror=unbanged-strict-patterns
-- For some reason the missing-home-modules warning
-- can be triggered for Internal.Helpers if the
-- following line is removed, cabal repl tests -O0 is
-- run, and :l Internal.Compiler.MAlonzo.Encode (say)
-- is executed in GHCi.
-Wno-missing-home-modules

if impl(ghc >= 8.6)
ghc-options: -Werror=inaccessible-code
-Werror=star-binder
-Werror=star-is-type
-- The following warning is an error in GHC >= 8.10.
if impl(ghc >= 8.6) && impl(ghc < 8.10)
ghc-options: -Werror=implicit-kind-vars

if impl(ghc >= 8.8)
ghc-options: -Werror=missed-extra-shared-lib

if impl(ghc >= 8.10)
ghc-options: -Werror=deriving-defaults
-Werror=redundant-record-wildcards
-Werror=unused-packages
-Werror=unused-record-wildcards

if impl(ghc >= 9.0)
ghc-options: -Werror=compat-unqualified-imports
-Werror=invalid-haddock
-- #6137: coverage checker works only sufficiently well from GHC 9.0
-Werror=incomplete-patterns
-Werror=incomplete-record-updates

-- ASR (2022-04-27). This warning was added in GHC 9.0.2, removed
-- from 9.2.1 and added back in 9.2.2.
if impl(ghc == 9.0.2)
ghc-options: -Werror=unicode-bidirectional-format-characters

if impl(ghc >= 9.2.2)
ghc-options: -Werror=redundant-bang-patterns
-Werror=unicode-bidirectional-format-characters
5 changes: 0 additions & 5 deletions stack-8.10.7.yaml
Original file line number Diff line number Diff line change
Expand Up @@ -2,11 +2,6 @@ resolver: lts-18.28
compiler: ghc-8.10.7
compiler-check: match-exact

# Local packages specified by relative directory name.
packages:
- '.'
- 'src/size-solver'

extra-deps:
- pqueue-1.5.0.0
- text-icu-0.8.0.2
Expand Down
6 changes: 0 additions & 6 deletions stack-8.6.5.yaml
Original file line number Diff line number Diff line change
Expand Up @@ -2,13 +2,7 @@ resolver: lts-14.27
compiler: ghc-8.6.5
compiler-check: match-exact

# Local packages specified by relative directory name.
packages:
- '.'
- 'src/size-solver'

extra-deps:
- QuickCheck-2.14.2
- STMonadTrans-0.4.3
- data-hash-0.2.0.1
- equivalence-0.3.4
Expand Down
5 changes: 0 additions & 5 deletions stack-8.8.4.yaml
Original file line number Diff line number Diff line change
Expand Up @@ -2,11 +2,6 @@ resolver: lts-16.31
compiler: ghc-8.8.4
compiler-check: match-exact

# Local packages specified by relative directory name.
packages:
- '.'
- 'src/size-solver'

extra-deps:
- QuickCheck-2.14.2
- pqueue-1.4.1.2
Expand Down
5 changes: 0 additions & 5 deletions stack-9.0.2.yaml
Original file line number Diff line number Diff line change
Expand Up @@ -2,11 +2,6 @@ resolver: lts-19.33
compiler: ghc-9.0.2
compiler-check: match-exact

# Local packages specified by relative directory name.
packages:
- '.'
- 'src/size-solver'

extra-deps:
- pqueue-1.5.0.0
- text-icu-0.8.0.2
Expand Down
5 changes: 0 additions & 5 deletions stack-9.2.8.yaml
Original file line number Diff line number Diff line change
Expand Up @@ -2,10 +2,5 @@ resolver: lts-20.26
compiler: ghc-9.2.8
compiler-check: match-exact

# Local packages specified by relative directory name.
packages:
- '.'
- 'src/size-solver'

extra-deps:
- pqueue-1.5.0.0
10 changes: 0 additions & 10 deletions stack-9.4.2.yaml
Original file line number Diff line number Diff line change
Expand Up @@ -2,11 +2,6 @@ resolver: ghc-9.4.2
compiler: ghc-9.4.2
compiler-check: match-exact

# Local packages specified by relative directory name.
packages:
- '.'
- 'src/size-solver'

flags:
mintty:
win32-2-13-1: false
Expand All @@ -16,7 +11,6 @@ extra-deps:
- Cabal-syntax-3.8.1.0
- ListLike-4.7.7
- OneTuple-0.3.1
- QuickCheck-2.14.2
- STMonadTrans-0.4.6
- StateVar-1.2.2
- Win32-2.12.0.1
Expand Down Expand Up @@ -100,10 +94,6 @@ extra-deps:
- stm-2.5.1.0
- strict-0.4.0.1
- tagged-0.8.6.1
- tasty-1.4.2.3
- tasty-hunit-0.10.0.3
- tasty-quickcheck-0.10.2
- tasty-silver-3.3.1.1
- template-haskell-2.19.0.0
- temporary-1.3
- terminfo-0.4.1.5
Expand Down
5 changes: 0 additions & 5 deletions stack-9.4.8.yaml
Original file line number Diff line number Diff line change
Expand Up @@ -2,11 +2,6 @@ resolver: lts-21.25
compiler: ghc-9.4.8
compiler-check: match-exact

# Local packages specified by relative directory name.
packages:
- '.'
- 'src/size-solver'

flags:
mintty:
win32-2-13-1: false
Expand Down

0 comments on commit 55b1c54

Please sign in to comment.