Agda.cabal 46 KB

123456789101112131415161718192021222324252627282930313233343536373839404142434445464748495051525354555657585960616263646566676869707172737475767778798081828384858687888990919293949596979899100101102103104105106107108109110111112113114115116117118119120121122123124125126127128129130131132133134135136137138139140141142143144145146147148149150151152153154155156157158159160161162163164165166167168169170171172173174175176177178179180181182183184185186187188189190191192193194195196197198199200201202203204205206207208209210211212213214215216217218219220221222223224225226227228229230231232233234235236237238239240241242243244245246247248249250251252253254255256257258259260261262263264265266267268269270271272273274275276277278279280281282283284285286287288289290291292293294295296297298299300301302303304305306307308309310311312313314315316317318319320321322323324325326327328329330331332333334335336337338339340341342343344345346347348349350351352353354355356357358359360361362363364365366367368369370371372373374375376377378379380381382383384385386387388389390391392393394395396397398399400401402403404405406407408409410411412413414415416417418419420421422423424425426427428429430431432433434435436437438439440441442443444445446447448449450451452453454455456457458459460461462463464465466467468469470471472473474475476477478479480481482483484485486487488489490491492493494495496497498499500501502503504505506507508509510511512513514515516517518519520521522523524525526527528529530531532533534535536537538539540541542543544545546547548549550551552553554555556557558559560561562563564565566567568569570571572573574575576577578579580581582583584585586587588589590591592593594595596597598599600601602603604605606607608609610611612613614615616617618619620621622623624625626627628629630631632633634635636637638639640641642643644645646647648649650651652653654655656657658659660661662663664665666667668669670671672673674675676677678679680681682683684685686687688689690691692693694695696697698699700701702703704705706707708709710711712713714715716717718719720721722723724725726727728729730731732733734735736737738739740741742743744745746747748749750751752753754755756757758759760761762763764765766767768769770771772773774775776777778779780781782783784785786787788789790791792793794795796797798799800801802803804805806807808809810811812813814815816817818819820821822823824825826827828829830831832833834835836837838839840841842843844845846847848849850851852853854855856857858859860861862863864865866867868869870871872873874875876877878879880881882883884885886887888889890891892893894895896897898899900901902903904905906907908909910911912913914915916917918919920921922923924925926927928929930931932933934935936937938939940941942943944945946947948949950951952953954955956957958959960961962963964965966967968969970971972973974975976977978979980981982983984985986987988989990991992993994995996997998999100010011002100310041005100610071008100910101011101210131014101510161017101810191020102110221023102410251026102710281029103010311032103310341035103610371038103910401041104210431044104510461047104810491050105110521053105410551056105710581059106010611062106310641065106610671068106910701071107210731074107510761077107810791080108110821083108410851086108710881089
  1. name: Agda
  2. version: 2.6.3
  3. cabal-version: >= 1.10
  4. build-type: Custom
  5. license: OtherLicense
  6. license-file: LICENSE
  7. copyright: (c) 2005-2021 The Agda Team.
  8. author: Ulf Norell and The Agda Team, see https://agda.readthedocs.io/en/latest/team.html
  9. maintainer: The Agda Team
  10. homepage: http://wiki.portal.chalmers.se/agda/
  11. bug-reports: https://github.com/agda/agda/issues
  12. category: Dependent types
  13. synopsis: A dependently typed functional programming language and proof assistant
  14. description:
  15. Agda is a dependently typed functional programming language: It has
  16. inductive families, which are similar to Haskell's GADTs, but they
  17. can be indexed by values and not just types. It also has
  18. parameterised modules, mixfix operators, Unicode characters, and an
  19. interactive Emacs interface (the type checker can assist in the
  20. development of your code).
  21. .
  22. Agda is also a proof assistant: It is an interactive system for
  23. writing and checking proofs. Agda is based on intuitionistic type
  24. theory, a foundational system for constructive mathematics developed
  25. by the Swedish logician Per Martin-Löf. It has many
  26. similarities with other proof assistants based on dependent types,
  27. such as Coq, Idris, Lean and NuPRL.
  28. .
  29. This package includes both a command-line program (agda) and an
  30. Emacs mode. If you want to use the Emacs mode you can set it up by
  31. running @agda-mode setup@ (see the README).
  32. .
  33. Note that the Agda package does not follow the package versioning
  34. policy, because it is not intended to be used by third-party
  35. packages.
  36. tested-with: GHC == 8.0.2
  37. GHC == 8.2.2
  38. GHC == 8.4.4
  39. GHC == 8.6.5
  40. GHC == 8.8.4
  41. GHC == 8.10.7
  42. GHC == 9.0.1
  43. GHC == 9.0.2
  44. GHC == 9.2.1
  45. extra-source-files: CHANGELOG.md
  46. README.md
  47. doc/release-notes/2.6.2.1.md
  48. doc/release-notes/2.6.2.md
  49. doc/release-notes/2.6.1.3.md
  50. doc/release-notes/2.6.1.2.md
  51. doc/release-notes/2.6.1.1.md
  52. doc/release-notes/2.6.1.md
  53. doc/release-notes/2.6.0.1.md
  54. doc/release-notes/2.6.0.md
  55. doc/release-notes/2.5.4.2.md
  56. doc/release-notes/2.5.4.1.md
  57. doc/release-notes/2.5.4.md
  58. doc/release-notes/2.5.3.md
  59. doc/release-notes/2.5.2.md
  60. doc/release-notes/2.5.1.2.md
  61. doc/release-notes/2.5.1.1.md
  62. doc/release-notes/2.5.1.md
  63. doc/release-notes/2.4.2.5.md
  64. doc/release-notes/2.4.2.4.md
  65. doc/release-notes/2.4.2.3.md
  66. doc/release-notes/2.4.2.2.md
  67. doc/release-notes/2.4.2.1.md
  68. doc/release-notes/2.4.2.md
  69. doc/release-notes/2.4.0.2.md
  70. doc/release-notes/2.4.0.1.md
  71. doc/release-notes/2.4.0.md
  72. doc/release-notes/2.3.2.2.md
  73. doc/release-notes/2.3.2.1.md
  74. doc/release-notes/2.3.2.md
  75. doc/release-notes/2.3.0.md
  76. doc/release-notes/2.2.10.md
  77. doc/release-notes/2.2.8.md
  78. doc/release-notes/2.2.6.md
  79. doc/release-notes/2.2.2.md
  80. doc/release-notes/2.2.4.md
  81. doc/release-notes/2.2.0.md
  82. -- Liang-Ting (2019-11-26): See Issues #4216
  83. -- doc/user-manual.pdf
  84. stack-8.0.2.yaml
  85. stack-8.2.2.yaml
  86. stack-8.4.4.yaml
  87. stack-8.6.5.yaml
  88. stack-8.8.4.yaml
  89. stack-8.10.7.yaml
  90. stack-9.0.1.yaml
  91. stack-9.0.2.yaml
  92. stack-9.2.1.yaml
  93. data-dir: src/data
  94. data-files: emacs-mode/*.el
  95. html/Agda.css
  96. html/highlight-hover.js
  97. JS/agda-rts.js
  98. latex/agda.sty
  99. latex/postprocess-latex.pl
  100. lib/prim/Agda/Builtin/Bool.agda
  101. lib/prim/Agda/Builtin/Char.agda
  102. lib/prim/Agda/Builtin/Char/Properties.agda
  103. lib/prim/Agda/Builtin/Coinduction.agda
  104. lib/prim/Agda/Builtin/Cubical/Path.agda
  105. lib/prim/Agda/Builtin/Cubical/Id.agda
  106. lib/prim/Agda/Builtin/Cubical/Sub.agda
  107. lib/prim/Agda/Builtin/Cubical/Glue.agda
  108. lib/prim/Agda/Builtin/Cubical/HCompU.agda
  109. lib/prim/Agda/Builtin/Equality.agda
  110. lib/prim/Agda/Builtin/Equality/Erase.agda
  111. lib/prim/Agda/Builtin/Equality/Rewrite.agda
  112. lib/prim/Agda/Builtin/Float.agda
  113. lib/prim/Agda/Builtin/Float/Properties.agda
  114. lib/prim/Agda/Builtin/FromNat.agda
  115. lib/prim/Agda/Builtin/FromNeg.agda
  116. lib/prim/Agda/Builtin/FromString.agda
  117. lib/prim/Agda/Builtin/IO.agda
  118. lib/prim/Agda/Builtin/Int.agda
  119. lib/prim/Agda/Builtin/List.agda
  120. lib/prim/Agda/Builtin/Maybe.agda
  121. lib/prim/Agda/Builtin/Nat.agda
  122. lib/prim/Agda/Builtin/Reflection.agda
  123. lib/prim/Agda/Builtin/Reflection/External.agda
  124. lib/prim/Agda/Builtin/Reflection/Properties.agda
  125. lib/prim/Agda/Builtin/Sigma.agda
  126. lib/prim/Agda/Builtin/Size.agda
  127. lib/prim/Agda/Builtin/Strict.agda
  128. lib/prim/Agda/Builtin/String.agda
  129. lib/prim/Agda/Builtin/String/Properties.agda
  130. lib/prim/Agda/Builtin/TrustMe.agda
  131. lib/prim/Agda/Builtin/Unit.agda
  132. lib/prim/Agda/Builtin/Word.agda
  133. lib/prim/Agda/Builtin/Word/Properties.agda
  134. lib/prim/Agda/Primitive.agda
  135. lib/prim/Agda/Primitive/Cubical.agda
  136. MAlonzo/src/MAlonzo/*.hs
  137. MAlonzo/src/MAlonzo/RTE/*.hs
  138. source-repository head
  139. type: git
  140. location: https://github.com/agda/agda.git
  141. source-repository this
  142. type: git
  143. location: https://github.com/agda/agda.git
  144. tag: v2.6.3
  145. flag cpphs
  146. default: False
  147. manual: True
  148. description: Use cpphs instead of cpp.
  149. flag debug
  150. default: False
  151. manual: True
  152. description:
  153. Enable debugging features that may slow Agda down.
  154. flag enable-cluster-counting
  155. default: False
  156. description:
  157. Enable the --count-clusters flag. (If enable-cluster-counting is
  158. False, then the --count-clusters flag triggers an error message.)
  159. flag optimise-heavily
  160. default: False
  161. description:
  162. Enable some expensive optimisations when compiling Agda.
  163. custom-setup
  164. setup-depends: base >= 4.9.0.0 && < 4.17
  165. , Cabal >= 1.24.0.0 && < 3.7
  166. , directory >= 1.2.6.2 && < 1.4
  167. , filepath >= 1.4.1.0 && < 1.5
  168. , process >= 1.4.2.0 && < 1.7
  169. library
  170. hs-source-dirs: src/full
  171. if flag(cpphs)
  172. -- We don't write an upper bound for cpphs because the
  173. -- `build-tools` field can not be modified in Hackage.
  174. build-tools: cpphs >= 1.20.9
  175. ghc-options: -pgmP cpphs -optP --cpp
  176. if flag(debug)
  177. cpp-options: -DDEBUG
  178. if flag(enable-cluster-counting)
  179. cpp-options: -DCOUNT_CLUSTERS
  180. build-depends: text-icu >= 0.7.1.0
  181. if os(windows)
  182. build-depends: Win32 >= 2.3.1.1 && < 2.13
  183. -- Agda cannot be built with GHC 8.6.1 due to a compiler bug, see
  184. -- Agda Issue #3344.
  185. if impl(ghc == 8.6.1)
  186. buildable: False
  187. -- Agda cannot be built with Windows and GHC 8.6.3 due to a compiler
  188. -- bug, see Agda Issue #3657.
  189. if os(windows) && impl(ghc == 8.6.3)
  190. buildable: False
  191. build-depends: aeson >= 1.1.2.0 && < 2.1
  192. , array >= 0.5.1.1 && < 0.6
  193. , async >= 2.2 && < 2.3
  194. , base >= 4.9.0.0 && < 4.17
  195. , binary >= 0.8.3.0 && < 0.9
  196. , blaze-html >= 0.8 && < 0.10
  197. , boxes >= 0.1.3 && < 0.2
  198. , bytestring >= 0.10.8.1 && < 0.12
  199. , case-insensitive >= 1.2.0.4 && < 1.3
  200. -- containers-0.5.11.0 is the first to contain IntSet.intersection
  201. , containers >= 0.5.11.0 && < 0.7
  202. , data-hash >= 0.2.0.0 && < 0.3
  203. , deepseq >= 1.4.2.0 && < 1.5
  204. , directory >= 1.2.6.2 && < 1.4
  205. , edit-distance >= 0.2.1.2 && < 0.3
  206. , equivalence >= 0.3.2 && < 0.5
  207. -- exceptions-0.8 instead of 0.10 because of stack
  208. , exceptions >= 0.8 && < 0.11
  209. , filepath >= 1.4.1.0 && < 1.5
  210. , gitrev >= 1.3.1 && < 2.0
  211. -- hashable 1.2.0.10 makes library-test 10x
  212. -- slower. The issue was fixed in hashable 1.2.1.0.
  213. -- https://github.com/tibbe/hashable/issues/57.
  214. , hashable >= 1.2.1.0 && < 1.5
  215. -- There is a "serious bug"
  216. -- (https://hackage.haskell.org/package/hashtables-1.2.0.2/changelog)
  217. -- in hashtables 1.2.0.0/1.2.0.1. This bug seems to
  218. -- have made Agda much slower (infinitely slower?) in
  219. -- some cases.
  220. , hashtables >= 1.2.0.2 && < 1.4
  221. , haskeline >= 0.7.2.3 && < 0.9
  222. -- monad-control-1.0.1.0 is the first to contain liftThrough
  223. , monad-control >= 1.0.1.0 && < 1.1
  224. -- mtl >= 2.2 && < 2.2.1 doesn't export Control.Monad.Except.
  225. -- Need mtl 2.2.2 for export of Control.Monad.IdentityT (ghc 8.2.2+)
  226. , mtl >= 2.2.1 && < 2.4
  227. , murmur-hash >= 0.1 && < 0.2
  228. , parallel >= 3.2.2.0 && < 3.3
  229. , pretty >= 1.1.3.3 && < 1.2
  230. , process >= 1.4.2.0 && < 1.7
  231. , regex-tdfa >= 1.3.1.0 && < 1.4
  232. , split >= 0.2.0.0 && < 0.2.4
  233. , stm >= 2.4.4 && < 2.6
  234. , strict >= 0.3.2 && < 0.5
  235. , template-haskell >= 2.11.0.0 && < 2.19
  236. , text >= 1.2.3.0 && < 2.1
  237. , time >= 1.6.0.1 && < 1.13
  238. , transformers >= 0.5 && < 0.7
  239. , unordered-containers >= 0.2.5.0 && < 0.3
  240. , uri-encode >= 1.5.0.4 && < 1.6
  241. , zlib == 0.6.*
  242. -- Andreas, 2022-02-02, issue #5659:
  243. -- Build failure with transformers-0.6.0.{0,1,2} and GHC 8.6.
  244. -- Transformers-0.6.0.3 might restored GHC 8.6 buildability.
  245. if impl(ghc == 8.6.*)
  246. build-depends: transformers < 0.6 || >= 0.6.0.3
  247. -- Andreas, 2021-03-10:
  248. -- All packages we depend upon should be mentioned in an unconditional
  249. -- build-depends field, but additional restrictions on their
  250. -- version for specific GHCs may be placed in conditionals.
  251. --
  252. -- The goal is to be able to make (e.g. when a new GHC comes out)
  253. -- revisions on hackage, e.g. relaxing upper bounds. This process
  254. -- currently does not support revising conditionals.
  255. -- ASR (2018-10-16).
  256. -- text-1.2.3.0 required for supporting GHC 8.4.1, 8.4.2 and
  257. -- 8.4.3. See Issue #3277.
  258. -- The other GHC versions can be restricted to >= 1.2.3.1.
  259. if impl(ghc < 8.4.1) || impl(ghc > 8.4.3)
  260. build-depends: text >= 1.2.3.1
  261. if impl(ghc >= 8.4)
  262. build-depends: ghc-compact == 0.1.*
  263. -- We don't write upper bounds for Alex nor Happy because the
  264. -- `build-tools` field can not be modified in Hackage. Agda doesn't
  265. -- build with Alex 3.2.0 and segfaults with 3.2.2.
  266. build-tools: alex >= 3.1.0 && < 3.2.0 || == 3.2.1 || >= 3.2.3
  267. , happy >= 1.19.4
  268. exposed-modules: Agda.Auto.Auto
  269. Agda.Auto.Options
  270. Agda.Auto.CaseSplit
  271. Agda.Auto.Convert
  272. Agda.Auto.NarrowingSearch
  273. Agda.Auto.SearchControl
  274. Agda.Auto.Syntax
  275. Agda.Auto.Typecheck
  276. Agda.Benchmarking
  277. Agda.Compiler.Backend
  278. Agda.Compiler.Builtin
  279. Agda.Compiler.CallCompiler
  280. Agda.Compiler.Common
  281. Agda.Compiler.JS.Compiler
  282. Agda.Compiler.JS.Syntax
  283. Agda.Compiler.JS.Substitution
  284. Agda.Compiler.JS.Pretty
  285. Agda.Compiler.MAlonzo.Coerce
  286. Agda.Compiler.MAlonzo.Compiler
  287. Agda.Compiler.MAlonzo.Encode
  288. Agda.Compiler.MAlonzo.HaskellTypes
  289. Agda.Compiler.MAlonzo.Misc
  290. Agda.Compiler.MAlonzo.Pragmas
  291. Agda.Compiler.MAlonzo.Pretty
  292. Agda.Compiler.MAlonzo.Primitives
  293. Agda.Compiler.MAlonzo.Strict
  294. Agda.Compiler.ToTreeless
  295. Agda.Compiler.Treeless.AsPatterns
  296. Agda.Compiler.Treeless.Builtin
  297. Agda.Compiler.Treeless.Compare
  298. Agda.Compiler.Treeless.EliminateDefaults
  299. Agda.Compiler.Treeless.EliminateLiteralPatterns
  300. Agda.Compiler.Treeless.Erase
  301. Agda.Compiler.Treeless.GuardsToPrims
  302. Agda.Compiler.Treeless.Identity
  303. Agda.Compiler.Treeless.NormalizeNames
  304. Agda.Compiler.Treeless.Pretty
  305. Agda.Compiler.Treeless.Simplify
  306. Agda.Compiler.Treeless.Subst
  307. Agda.Compiler.Treeless.Uncase
  308. Agda.Compiler.Treeless.Unused
  309. Agda.ImpossibleTest
  310. Agda.Interaction.AgdaTop
  311. Agda.Interaction.Base
  312. Agda.Interaction.BasicOps
  313. Agda.Interaction.SearchAbout
  314. Agda.Interaction.CommandLine
  315. Agda.Interaction.EmacsCommand
  316. Agda.Interaction.EmacsTop
  317. Agda.Interaction.ExitCode
  318. Agda.Interaction.JSONTop
  319. Agda.Interaction.JSON
  320. Agda.Interaction.FindFile
  321. Agda.Interaction.Highlighting.Common
  322. Agda.Interaction.Highlighting.Dot
  323. Agda.Interaction.Highlighting.Emacs
  324. Agda.Interaction.Highlighting.FromAbstract
  325. Agda.Interaction.Highlighting.Generate
  326. Agda.Interaction.Highlighting.HTML
  327. Agda.Interaction.Highlighting.JSON
  328. Agda.Interaction.Highlighting.Precise
  329. Agda.Interaction.Highlighting.Range
  330. Agda.Interaction.Highlighting.Vim
  331. Agda.Interaction.Highlighting.LaTeX
  332. Agda.Interaction.Imports
  333. Agda.Interaction.InteractionTop
  334. Agda.Interaction.Response
  335. Agda.Interaction.MakeCase
  336. Agda.Interaction.Monad
  337. Agda.Interaction.Library
  338. Agda.Interaction.Library.Base
  339. Agda.Interaction.Library.Parse
  340. Agda.Interaction.Options
  341. Agda.Interaction.Options.Help
  342. Agda.Interaction.Options.Lenses
  343. Agda.Interaction.Options.Warnings
  344. Agda.Main
  345. Agda.Syntax.Abstract.Name
  346. Agda.Syntax.Abstract.Pattern
  347. Agda.Syntax.Abstract.PatternSynonyms
  348. Agda.Syntax.Abstract.Pretty
  349. Agda.Syntax.Abstract.Views
  350. Agda.Syntax.Abstract
  351. Agda.Syntax.Builtin
  352. Agda.Syntax.Common
  353. Agda.Syntax.Concrete.Attribute
  354. Agda.Syntax.Concrete.Definitions
  355. Agda.Syntax.Concrete.Definitions.Errors
  356. Agda.Syntax.Concrete.Definitions.Monad
  357. Agda.Syntax.Concrete.Definitions.Types
  358. Agda.Syntax.Concrete.Fixity
  359. Agda.Syntax.Concrete.Generic
  360. Agda.Syntax.Concrete.Glyph
  361. Agda.Syntax.Concrete.Name
  362. Agda.Syntax.Concrete.Operators.Parser
  363. Agda.Syntax.Concrete.Operators.Parser.Monad
  364. Agda.Syntax.Concrete.Operators
  365. Agda.Syntax.Concrete.Pattern
  366. Agda.Syntax.Concrete.Pretty
  367. Agda.Syntax.Concrete
  368. Agda.Syntax.DoNotation
  369. Agda.Syntax.Fixity
  370. Agda.Syntax.IdiomBrackets
  371. Agda.Syntax.Info
  372. Agda.Syntax.Internal
  373. Agda.Syntax.Internal.Blockers
  374. Agda.Syntax.Internal.Defs
  375. Agda.Syntax.Internal.Elim
  376. Agda.Syntax.Internal.Generic
  377. Agda.Syntax.Internal.MetaVars
  378. Agda.Syntax.Internal.Names
  379. Agda.Syntax.Internal.Pattern
  380. Agda.Syntax.Internal.SanityCheck
  381. Agda.Syntax.Literal
  382. Agda.Syntax.Notation
  383. Agda.Syntax.Parser.Alex
  384. Agda.Syntax.Parser.Comments
  385. Agda.Syntax.Parser.Layout
  386. Agda.Syntax.Parser.LexActions
  387. Agda.Syntax.Parser.Lexer
  388. Agda.Syntax.Parser.Literate
  389. Agda.Syntax.Parser.LookAhead
  390. Agda.Syntax.Parser.Monad
  391. Agda.Syntax.Parser.Parser
  392. Agda.Syntax.Parser.StringLiterals
  393. Agda.Syntax.Parser.Tokens
  394. Agda.Syntax.Parser
  395. Agda.Syntax.Position
  396. Agda.Syntax.Reflected
  397. Agda.Syntax.Scope.Base
  398. Agda.Syntax.Scope.Monad
  399. Agda.Syntax.Translation.AbstractToConcrete
  400. Agda.Syntax.Translation.ConcreteToAbstract
  401. Agda.Syntax.Translation.InternalToAbstract
  402. Agda.Syntax.Translation.ReflectedToAbstract
  403. Agda.Syntax.Treeless
  404. Agda.Termination.CallGraph
  405. Agda.Termination.CallMatrix
  406. Agda.Termination.CutOff
  407. Agda.Termination.Monad
  408. Agda.Termination.Order
  409. Agda.Termination.RecCheck
  410. Agda.Termination.SparseMatrix
  411. Agda.Termination.Semiring
  412. Agda.Termination.TermCheck
  413. Agda.Termination.Termination
  414. Agda.TheTypeChecker
  415. Agda.TypeChecking.Abstract
  416. Agda.TypeChecking.CheckInternal
  417. Agda.TypeChecking.CompiledClause
  418. Agda.TypeChecking.CompiledClause.Compile
  419. Agda.TypeChecking.CompiledClause.Match
  420. Agda.TypeChecking.Constraints
  421. Agda.TypeChecking.Conversion
  422. Agda.TypeChecking.Conversion.Pure
  423. Agda.TypeChecking.Coverage
  424. Agda.TypeChecking.Coverage.Match
  425. Agda.TypeChecking.Coverage.SplitTree
  426. Agda.TypeChecking.Coverage.SplitClause
  427. Agda.TypeChecking.Coverage.Cubical
  428. Agda.TypeChecking.Datatypes
  429. Agda.TypeChecking.DeadCode
  430. Agda.TypeChecking.DisplayForm
  431. Agda.TypeChecking.DropArgs
  432. Agda.TypeChecking.Empty
  433. Agda.TypeChecking.EtaContract
  434. Agda.TypeChecking.EtaExpand
  435. Agda.TypeChecking.Errors
  436. Agda.TypeChecking.Free
  437. Agda.TypeChecking.Free.Lazy
  438. Agda.TypeChecking.Free.Precompute
  439. Agda.TypeChecking.Free.Reduce
  440. Agda.TypeChecking.Forcing
  441. Agda.TypeChecking.Functions
  442. Agda.TypeChecking.Generalize
  443. Agda.TypeChecking.IApplyConfluence
  444. Agda.TypeChecking.Implicit
  445. Agda.TypeChecking.Injectivity
  446. Agda.TypeChecking.Inlining
  447. Agda.TypeChecking.InstanceArguments
  448. Agda.TypeChecking.Irrelevance
  449. Agda.TypeChecking.Level
  450. Agda.TypeChecking.LevelConstraints
  451. Agda.TypeChecking.Lock
  452. Agda.TypeChecking.Level.Solve
  453. Agda.TypeChecking.MetaVars
  454. Agda.TypeChecking.MetaVars.Mention
  455. Agda.TypeChecking.MetaVars.Occurs
  456. Agda.TypeChecking.Monad.Base
  457. Agda.TypeChecking.Monad.Benchmark
  458. Agda.TypeChecking.Monad.Builtin
  459. Agda.TypeChecking.Monad.Caching
  460. Agda.TypeChecking.Monad.Closure
  461. Agda.TypeChecking.Monad.Constraints
  462. Agda.TypeChecking.Monad.Context
  463. Agda.TypeChecking.Monad.Debug
  464. Agda.TypeChecking.Monad.Env
  465. Agda.TypeChecking.Monad.Imports
  466. Agda.TypeChecking.Monad.MetaVars
  467. Agda.TypeChecking.Monad.Mutual
  468. Agda.TypeChecking.Monad.Open
  469. Agda.TypeChecking.Monad.Options
  470. Agda.TypeChecking.Monad.Pure
  471. Agda.TypeChecking.Monad.Signature
  472. Agda.TypeChecking.Monad.SizedTypes
  473. Agda.TypeChecking.Monad.State
  474. Agda.TypeChecking.Monad.Statistics
  475. Agda.TypeChecking.Monad.Trace
  476. Agda.TypeChecking.Monad
  477. Agda.TypeChecking.Names
  478. Agda.TypeChecking.Patterns.Abstract
  479. Agda.TypeChecking.Patterns.Internal
  480. Agda.TypeChecking.Patterns.Match
  481. Agda.TypeChecking.Polarity
  482. Agda.TypeChecking.Positivity
  483. Agda.TypeChecking.Positivity.Occurrence
  484. Agda.TypeChecking.Pretty
  485. Agda.TypeChecking.Pretty.Call
  486. Agda.TypeChecking.Pretty.Constraint
  487. Agda.TypeChecking.Pretty.Warning
  488. Agda.TypeChecking.Primitive
  489. Agda.TypeChecking.Primitive.Base
  490. Agda.TypeChecking.Primitive.Cubical
  491. Agda.TypeChecking.ProjectionLike
  492. Agda.TypeChecking.Quote
  493. Agda.TypeChecking.ReconstructParameters
  494. Agda.TypeChecking.RecordPatterns
  495. Agda.TypeChecking.Records
  496. Agda.TypeChecking.Reduce
  497. Agda.TypeChecking.Reduce.Fast
  498. Agda.TypeChecking.Reduce.Monad
  499. Agda.TypeChecking.Rewriting
  500. Agda.TypeChecking.Rewriting.Clause
  501. Agda.TypeChecking.Rewriting.Confluence
  502. Agda.TypeChecking.Rewriting.NonLinMatch
  503. Agda.TypeChecking.Rewriting.NonLinPattern
  504. Agda.TypeChecking.Rules.Application
  505. Agda.TypeChecking.Rules.Builtin
  506. Agda.TypeChecking.Rules.Builtin.Coinduction
  507. Agda.TypeChecking.Rules.Data
  508. Agda.TypeChecking.Rules.Decl
  509. Agda.TypeChecking.Rules.Def
  510. Agda.TypeChecking.Rules.Display
  511. Agda.TypeChecking.Rules.LHS
  512. Agda.TypeChecking.Rules.LHS.Implicit
  513. Agda.TypeChecking.Rules.LHS.Problem
  514. Agda.TypeChecking.Rules.LHS.ProblemRest
  515. Agda.TypeChecking.Rules.LHS.Unify
  516. Agda.TypeChecking.Rules.LHS.Unify.Types
  517. Agda.TypeChecking.Rules.LHS.Unify.LeftInverse
  518. Agda.TypeChecking.Rules.Record
  519. Agda.TypeChecking.Rules.Term
  520. Agda.TypeChecking.Serialise
  521. Agda.TypeChecking.Serialise.Base
  522. Agda.TypeChecking.Serialise.Instances
  523. Agda.TypeChecking.Serialise.Instances.Abstract
  524. Agda.TypeChecking.Serialise.Instances.Common
  525. Agda.TypeChecking.Serialise.Instances.Compilers
  526. Agda.TypeChecking.Serialise.Instances.Highlighting
  527. Agda.TypeChecking.Serialise.Instances.Internal
  528. Agda.TypeChecking.Serialise.Instances.Errors
  529. Agda.TypeChecking.SizedTypes
  530. Agda.TypeChecking.SizedTypes.Solve
  531. Agda.TypeChecking.SizedTypes.Syntax
  532. Agda.TypeChecking.SizedTypes.Utils
  533. Agda.TypeChecking.SizedTypes.WarshallSolver
  534. Agda.TypeChecking.Sort
  535. Agda.TypeChecking.Substitute
  536. Agda.TypeChecking.Substitute.Class
  537. Agda.TypeChecking.Substitute.DeBruijn
  538. Agda.TypeChecking.SyntacticEquality
  539. Agda.TypeChecking.Telescope
  540. Agda.TypeChecking.Telescope.Path
  541. Agda.TypeChecking.Unquote
  542. Agda.TypeChecking.Warnings
  543. Agda.TypeChecking.With
  544. Agda.Utils.AffineHole
  545. Agda.Utils.Applicative
  546. Agda.Utils.AssocList
  547. Agda.Utils.Bag
  548. Agda.Utils.Benchmark
  549. Agda.Utils.BiMap
  550. Agda.Utils.CallStack
  551. Agda.Utils.Char
  552. Agda.Utils.Cluster
  553. Agda.Utils.Empty
  554. Agda.Utils.Environment
  555. Agda.Utils.Either
  556. Agda.Utils.Fail
  557. Agda.Utils.Favorites
  558. Agda.Utils.FileName
  559. Agda.Utils.Float
  560. Agda.Utils.Functor
  561. Agda.Utils.Function
  562. Agda.Utils.Graph.AdjacencyMap.Unidirectional
  563. Agda.Utils.Graph.TopSort
  564. Agda.Utils.Hash
  565. Agda.Utils.Haskell.Syntax
  566. Agda.Utils.Impossible
  567. Agda.Utils.IndexedList
  568. Agda.Utils.IntSet.Infinite
  569. Agda.Utils.IO
  570. Agda.Utils.IO.Binary
  571. Agda.Utils.IO.Directory
  572. Agda.Utils.IO.TempFile
  573. Agda.Utils.IO.UTF8
  574. Agda.Utils.IORef
  575. Agda.Utils.Lens
  576. Agda.Utils.Lens.Examples
  577. Agda.Utils.List
  578. Agda.Utils.List1
  579. Agda.Utils.List2
  580. Agda.Utils.ListT
  581. Agda.Utils.Map
  582. Agda.Utils.Maybe
  583. Agda.Utils.Maybe.Strict
  584. Agda.Utils.Memo
  585. Agda.Utils.Monad
  586. Agda.Utils.Monoid
  587. Agda.Utils.Null
  588. Agda.Utils.Parser.MemoisedCPS
  589. Agda.Utils.PartialOrd
  590. Agda.Utils.Permutation
  591. Agda.Utils.Pointer
  592. Agda.Utils.POMonoid
  593. Agda.Utils.Pretty
  594. Agda.Utils.ProfileOptions
  595. Agda.Utils.RangeMap
  596. Agda.Utils.SemiRing
  597. Agda.Utils.Semigroup
  598. Agda.Utils.Singleton
  599. Agda.Utils.Size
  600. Agda.Utils.SmallSet
  601. Agda.Utils.String
  602. Agda.Utils.Suffix
  603. Agda.Utils.Three
  604. Agda.Utils.Time
  605. Agda.Utils.Trie
  606. Agda.Utils.Tuple
  607. Agda.Utils.TypeLevel
  608. Agda.Utils.TypeLits
  609. Agda.Utils.Update
  610. Agda.Utils.VarSet
  611. Agda.Utils.Warshall
  612. Agda.Utils.WithDefault
  613. Agda.Utils.Zipper
  614. Agda.Version
  615. Agda.VersionCommit
  616. other-modules: Paths_Agda
  617. Agda.Interaction.Highlighting.Dot.Backend
  618. Agda.Interaction.Highlighting.Dot.Base
  619. Agda.Interaction.Highlighting.HTML.Backend
  620. Agda.Interaction.Highlighting.HTML.Base
  621. Agda.Interaction.Highlighting.LaTeX.Backend
  622. Agda.Interaction.Highlighting.LaTeX.Base
  623. Agda.Interaction.Options.Base
  624. Agda.Interaction.Options.HasOptions
  625. Agda.Utils.CallStack.Base
  626. Agda.Utils.CallStack.Pretty
  627. if flag(optimise-heavily)
  628. ghc-options: -fexpose-all-unfoldings
  629. -fspecialise-aggressively
  630. -- NOTE: If adding flags, also add to `.ghci-8.0`
  631. if impl(ghc <= 8.0.2)
  632. ghc-options: -fprint-potential-instances
  633. -- Initially, we disable all the warnings.
  634. -w
  635. -Werror
  636. -- This option must be the first one after disabling the
  637. -- warnings. See Issue #2094.
  638. -Wunrecognised-warning-flags
  639. -Wdeprecated-flags
  640. -Wderiving-typeable
  641. -Wdodgy-exports
  642. -Wdodgy-foreign-imports
  643. -Wdodgy-imports
  644. -Wduplicate-exports
  645. -Wempty-enumerations
  646. -Widentities
  647. -Wincomplete-patterns
  648. -Winline-rule-shadowing
  649. -Wmissing-fields
  650. -Wmissing-methods
  651. -Wmissing-pattern-synonym-signatures
  652. -Wmissing-signatures
  653. -Wnoncanonical-monad-instances
  654. -Wnoncanonical-monoid-instances
  655. -Woverflowed-literals
  656. -Woverlapping-patterns
  657. -Wsemigroup
  658. -Wtabs
  659. -Wtyped-holes
  660. -Wunrecognised-pragmas
  661. -Wunticked-promoted-constructors
  662. -Wunused-do-bind
  663. -Wunused-foralls
  664. -Wwarnings-deprecations
  665. -Wwrong-do-bind
  666. else
  667. ghc-options: -fprint-potential-instances
  668. -Werror=unrecognised-warning-flags
  669. -Werror=deprecated-flags
  670. -Werror=deriving-typeable
  671. -Werror=dodgy-exports
  672. -Werror=dodgy-foreign-imports
  673. -Werror=dodgy-imports
  674. -Werror=duplicate-exports
  675. -Werror=empty-enumerations
  676. -Werror=identities
  677. -Werror=incomplete-patterns
  678. -Werror=inline-rule-shadowing
  679. -Werror=missing-fields
  680. -Werror=missing-methods
  681. -Werror=missing-pattern-synonym-signatures
  682. -Werror=missing-signatures
  683. -Werror=noncanonical-monad-instances
  684. -Werror=noncanonical-monoid-instances
  685. -Werror=overflowed-literals
  686. -Werror=overlapping-patterns
  687. -Werror=semigroup
  688. -Werror=tabs
  689. -Werror=typed-holes
  690. -Werror=unrecognised-pragmas
  691. -Werror=unticked-promoted-constructors
  692. -Werror=unused-do-bind
  693. -Werror=unused-foralls
  694. -Werror=warnings-deprecations
  695. -Werror=wrong-do-bind
  696. -- NOTE: If adding or removing flags, also change `.ghci-8.2`
  697. if impl(ghc >= 8.2)
  698. ghc-options: -Wcpp-undef
  699. -- ASR TODO (2017-07-23): `make haddock` fails when
  700. -- this flag is on.
  701. -- -Wmissing-home-modules
  702. -Werror=simplifiable-class-constraints
  703. -Werror=unbanged-strict-patterns
  704. -- NOTE: If adding or removing flags, also change `.ghci-8.6`
  705. if impl(ghc >= 8.6)
  706. ghc-options: -Werror=inaccessible-code
  707. -Werror=star-binder
  708. -Werror=star-is-type
  709. -- The following warning is an error in GHC >= 8.10.
  710. if impl(ghc >= 8.6) && impl(ghc < 8.10)
  711. ghc-options: -Werror=implicit-kind-vars
  712. -- NOTE: If adding or removing flags, also change `.ghci-8.8`
  713. if impl(ghc >= 8.8)
  714. ghc-options: -Werror=missed-extra-shared-lib
  715. -- NOTE: If adding or removing flags, also change `.ghci-8.10`
  716. if impl(ghc >= 8.10)
  717. ghc-options: -Werror=deriving-defaults
  718. -Werror=redundant-record-wildcards
  719. -Werror=unused-packages
  720. -Werror=unused-record-wildcards
  721. -- NOTE: If adding or removing flags, also change `.ghci-9.0`
  722. if impl(ghc >= 9.0)
  723. ghc-options: -Werror=invalid-haddock
  724. ghc-prof-options: -fprof-auto
  725. default-language: Haskell2010
  726. -- NOTE: If adding or removing default extensions, also change:
  727. -- .ghci-8.0
  728. -- .hlint.yaml
  729. -- This should also use the same extensions as the `test-suite` target below.
  730. default-extensions: BangPatterns
  731. , ConstraintKinds
  732. --L-T Chen (2019-07-15):
  733. -- Enabling DataKinds only locally makes the compile time
  734. -- slightly shorter, see PR #3920.
  735. --, DataKinds
  736. , DefaultSignatures
  737. , DeriveDataTypeable
  738. , DeriveFoldable
  739. , DeriveFunctor
  740. , DeriveGeneric
  741. , DeriveTraversable
  742. , ExistentialQuantification
  743. , FlexibleContexts
  744. , FlexibleInstances
  745. , FunctionalDependencies
  746. , GeneralizedNewtypeDeriving
  747. , InstanceSigs
  748. , LambdaCase
  749. , MultiParamTypeClasses
  750. , MultiWayIf
  751. , NamedFieldPuns
  752. , OverloadedStrings
  753. , PatternSynonyms
  754. , RankNTypes
  755. , RecordWildCards
  756. , ScopedTypeVariables
  757. , StandaloneDeriving
  758. , TupleSections
  759. , TypeFamilies
  760. , TypeSynonymInstances
  761. executable agda
  762. hs-source-dirs: src/main
  763. main-is: Main.hs
  764. build-depends: Agda
  765. -- A version range on Agda generates a warning with
  766. -- some versions of Cabal and GHC
  767. -- (e.g. cabal-install version 1.24.0.2 compiled
  768. -- using version 1.24.2.0 of the Cabal library and
  769. -- GHC 8.2.1 RC1).
  770. -- Nothing is used from the following package,
  771. -- except for the Prelude.
  772. , base
  773. default-language: Haskell2010
  774. -- If someone installs Agda with the setuid bit set, then the
  775. -- presence of +RTS may be a security problem (see GHC bug #3910).
  776. -- However, we sometimes recommend people to use +RTS to control
  777. -- Agda's memory usage, so we want this functionality enabled by
  778. -- default.
  779. -- The threaded RTS by default starts a major GC after a program has
  780. -- been idle for 0.3 s. This feature turned out to be annoying, so
  781. -- the idle GC is now by default turned off (-I0).
  782. ghc-options: -threaded -rtsopts
  783. "-with-rtsopts=-M3.5G -I0"
  784. executable agda-mode
  785. hs-source-dirs: src/agda-mode
  786. main-is: Main.hs
  787. other-modules: Paths_Agda
  788. build-depends: base >= 4.9.0.0 && < 4.17
  789. , directory >= 1.2.6.2 && < 1.4
  790. , filepath >= 1.4.1.0 && < 1.5
  791. , process >= 1.4.2.0 && < 1.7
  792. default-language: Haskell2010
  793. -- Cabal testsuite integration has some serious bugs, but we
  794. -- can still make it work. See also:
  795. -- https://github.com/haskell/cabal/issues/1938
  796. -- https://github.com/haskell/cabal/issues/2214
  797. -- https://github.com/haskell/cabal/issues/1953
  798. --
  799. -- This test suite should only be run using the Makefile.
  800. -- The Makefile sets up the required environment,
  801. -- executing the tests using cabal directly is almost
  802. -- guaranteed to fail. See also Issue 1490.
  803. test-suite agda-tests
  804. type: exitcode-stdio-1.0
  805. hs-source-dirs: test/
  806. main-is: Main.hs
  807. other-modules: Bugs.Tests
  808. , Compiler.Tests
  809. , Fail.Tests
  810. , Interactive.Tests
  811. , Internal.Compiler.MAlonzo.Encode
  812. , Internal.Helpers
  813. , Internal.Interaction.Highlighting.Precise
  814. , Internal.Interaction.Highlighting.Range
  815. , Internal.Interaction.Library
  816. , Internal.Interaction.Options
  817. , Internal.Syntax.Abstract.Name
  818. , Internal.Syntax.Common
  819. , Internal.Syntax.Concrete.Name
  820. , Internal.Syntax.Internal
  821. , Internal.Syntax.Parser.Parser
  822. , Internal.Syntax.Position
  823. , Internal.Termination.CallGraph
  824. , Internal.Termination.CallMatrix
  825. , Internal.Termination.Order
  826. , Internal.Termination.Semiring
  827. , Internal.Termination.SparseMatrix
  828. , Internal.Termination.Termination
  829. , Internal.Tests
  830. , Internal.TypeChecking
  831. , Internal.TypeChecking.Free
  832. , Internal.TypeChecking.Free.Lazy
  833. , Internal.TypeChecking.Generators
  834. , Internal.TypeChecking.Irrelevance
  835. , Internal.TypeChecking.Monad.Base
  836. , Internal.TypeChecking.Positivity
  837. , Internal.TypeChecking.Positivity.Occurrence
  838. , Internal.TypeChecking.Rules.LHS.Problem
  839. , Internal.TypeChecking.SizedTypes
  840. , Internal.TypeChecking.SizedTypes.Syntax
  841. , Internal.TypeChecking.SizedTypes.WarshallSolver
  842. , Internal.TypeChecking.Substitute
  843. , Internal.Utils.AssocList
  844. , Internal.Utils.Bag
  845. , Internal.Utils.BiMap
  846. , Internal.Utils.Cluster
  847. , Internal.Utils.Either
  848. , Internal.Utils.Favorites
  849. , Internal.Utils.FileName
  850. , Internal.Utils.Graph.AdjacencyMap.Unidirectional
  851. , Internal.Utils.IntSet
  852. , Internal.Utils.List
  853. , Internal.Utils.ListT
  854. , Internal.Utils.Maybe.Strict
  855. , Internal.Utils.Monoid
  856. , Internal.Utils.NonEmptyList
  857. , Internal.Utils.PartialOrd
  858. , Internal.Utils.Permutation
  859. , Internal.Utils.RangeMap
  860. , Internal.Utils.SmallSet
  861. , Internal.Utils.Three
  862. , Internal.Utils.Trie
  863. , Internal.Utils.Warshall
  864. , LaTeXAndHTML.Tests
  865. , LibSucceed.Tests
  866. , Succeed.Tests
  867. , UserManual.Tests
  868. , Utils
  869. -- Andreas, 2021-08-26, see https://github.com/haskell/cabal/issues/7577
  870. -- Since 'agda-tests' wants to call 'agda', we have to add it here,
  871. -- should we want to run 'cabal test'.
  872. build-tool-depends: Agda:agda
  873. build-depends: Agda
  874. , array
  875. , base
  876. , bytestring
  877. , containers
  878. , directory
  879. , filepath
  880. , filemanip >= 0.3.6.3 && < 0.4
  881. , mtl
  882. , process
  883. , process-extras >= 0.3.0 && < 0.3.4 || >= 0.4.1.3 && < 0.5 || >= 0.7.1 && < 0.8
  884. , QuickCheck >= 2.14.1 && < 2.15
  885. , regex-tdfa
  886. , strict >= 0.3.2 && < 0.5
  887. , tasty >= 1.1.0.4 && < 1.5
  888. , tasty-hunit >= 0.9.2 && < 0.11
  889. , tasty-quickcheck >= 0.9.2 && < 0.11
  890. -- tasty-silver 3.1.13 has option --ansi-tricks=false
  891. -- NB: tasty-silver 3.2 requires tasty >= 1.4
  892. -- tasty-silver < 3.3 does not work interactively under Windows
  893. , tasty-silver >= 3.1.13 && < 3.4
  894. , temporary >= 1.2.0.3 && < 1.4
  895. , text
  896. , unix-compat >= 0.4.3.1 && < 0.6
  897. , unordered-containers >= 0.2.5.0 && < 0.3
  898. , uri-encode
  899. -- Andreas (2021-10-11): tasty-silver < 3.3 does not work interactively under Windows
  900. if os(windows)
  901. build-depends: tasty-silver >= 3.3
  902. default-language: Haskell2010
  903. -- NOTE: If adding or removing default extensions, also change:
  904. -- .ghci-8.0
  905. -- .hlint.yaml
  906. -- This should also use the same extensions as the `library` target above.
  907. default-extensions: BangPatterns
  908. , ConstraintKinds
  909. --L-T Chen (2019-07-15):
  910. -- Enabling DataKinds only locally makes the compile time
  911. -- slightly shorter, see PR #3920.
  912. --, DataKinds
  913. , DefaultSignatures
  914. , DeriveDataTypeable
  915. , DeriveFoldable
  916. , DeriveFunctor
  917. , DeriveGeneric
  918. , DeriveTraversable
  919. , ExistentialQuantification
  920. , FlexibleContexts
  921. , FlexibleInstances
  922. , FunctionalDependencies
  923. , GeneralizedNewtypeDeriving
  924. , InstanceSigs
  925. , LambdaCase
  926. , MultiParamTypeClasses
  927. , MultiWayIf
  928. , NamedFieldPuns
  929. , OverloadedStrings
  930. , PatternSynonyms
  931. , RankNTypes
  932. , RecordWildCards
  933. , ScopedTypeVariables
  934. , StandaloneDeriving
  935. , TupleSections
  936. , TypeFamilies
  937. , TypeSynonymInstances
  938. if flag(optimise-heavily)
  939. ghc-options: -fexpose-all-unfoldings
  940. -fspecialise-aggressively
  941. -- NOTE: If adding or removing flags, also change `.ghci-8.0`
  942. if impl(ghc <= 8.0.2)
  943. ghc-options: -threaded
  944. -- Initially, we disable all the warnings.
  945. -w
  946. -Werror
  947. -- This option must be the first one after disabling the
  948. -- warnings. See Issue #2094.
  949. -Wunrecognised-warning-flags
  950. -Wdeprecated-flags
  951. -Wderiving-typeable
  952. -Wdodgy-exports
  953. -Wdodgy-foreign-imports
  954. -Wdodgy-imports
  955. -Wduplicate-exports
  956. -Wempty-enumerations
  957. -Widentities
  958. -Wincomplete-patterns
  959. -Winline-rule-shadowing
  960. -Wmissing-fields
  961. -Wmissing-methods
  962. -Wmissing-pattern-synonym-signatures
  963. -Wmissing-signatures
  964. -Wnoncanonical-monad-instances
  965. -Wnoncanonical-monoid-instances
  966. -Woverflowed-literals
  967. -Woverlapping-patterns
  968. -Wsemigroup
  969. -Wtabs
  970. -Wtyped-holes
  971. -Wunrecognised-pragmas
  972. -Wunticked-promoted-constructors
  973. -Wunused-do-bind
  974. -Wunused-foralls
  975. -Wwarnings-deprecations
  976. -Wwrong-do-bind
  977. else
  978. ghc-options: -threaded
  979. -Werror=unrecognised-warning-flags
  980. -Werror=deprecated-flags
  981. -Werror=deriving-typeable
  982. -Werror=dodgy-exports
  983. -Werror=dodgy-foreign-imports
  984. -Werror=dodgy-imports
  985. -Werror=duplicate-exports
  986. -Werror=empty-enumerations
  987. -Werror=identities
  988. -Werror=incomplete-patterns
  989. -Werror=inline-rule-shadowing
  990. -Werror=missing-fields
  991. -Werror=missing-methods
  992. -Werror=missing-pattern-synonym-signatures
  993. -Werror=missing-signatures
  994. -Werror=noncanonical-monad-instances
  995. -Werror=noncanonical-monoid-instances
  996. -Werror=overflowed-literals
  997. -Werror=overlapping-patterns
  998. -Werror=semigroup
  999. -Werror=tabs
  1000. -Werror=typed-holes
  1001. -Werror=unrecognised-pragmas
  1002. -Werror=unticked-promoted-constructors
  1003. -Werror=unused-do-bind
  1004. -Werror=unused-foralls
  1005. -Werror=warnings-deprecations
  1006. -Werror=wrong-do-bind
  1007. -- ASR (2017-04-11). TODO: Using -Werror=missing-home-modules generates an
  1008. -- error.
  1009. -- NOTE: If adding or removing flags, also change `.ghci-8.2`
  1010. if impl(ghc >= 8.2)
  1011. ghc-options: -Werror=cpp-undef
  1012. -Werror=simplifiable-class-constraints
  1013. -Werror=unbanged-strict-patterns
  1014. -- NOTE: If adding or removing flags, also change `.ghci-8.6`
  1015. if impl(ghc >= 8.6)
  1016. ghc-options: -Werror=inaccessible-code
  1017. -Werror=star-binder
  1018. -Werror=star-is-type
  1019. -- The following warning is an error in GHC >= 8.10.
  1020. if impl(ghc >= 8.6) && impl(ghc < 8.10)
  1021. ghc-options: -Werror=implicit-kind-vars
  1022. -- NOTE: If adding or removing flags, also change `.ghci-8.8`
  1023. if impl(ghc >= 8.8)
  1024. ghc-options: -Werror=missed-extra-shared-lib
  1025. -- NOTE: If adding or removing flags, also change `.ghci-8.10`
  1026. if impl(ghc >= 8.10)
  1027. ghc-options: -Werror=deriving-defaults
  1028. -Werror=redundant-record-wildcards
  1029. -Werror=unused-packages
  1030. -Werror=unused-record-wildcards
  1031. -- NOTE: If adding or removing flags, also change `.ghci-9.0`
  1032. if impl(ghc >= 9.0)
  1033. ghc-options: -Werror=compat-unqualified-imports
  1034. -Werror=invalid-haddock