Agda.cabal 46 KB

12345678910111213141516171819202122232425262728293031323334353637383940414243444546474849505152535455565758596061626364656667686970717273747576777879808182838485868788899091929394959697989910010110210310410510610710810911011111211311411511611711811912012112212312412512612712812913013113213313413513613713813914014114214314414514614714814915015115215315415515615715815916016116216316416516616716816917017117217317417517617717817918018118218318418518618718818919019119219319419519619719819920020120220320420520620720820921021121221321421521621721821922022122222322422522622722822923023123223323423523623723823924024124224324424524624724824925025125225325425525625725825926026126226326426526626726826927027127227327427527627727827928028128228328428528628728828929029129229329429529629729829930030130230330430530630730830931031131231331431531631731831932032132232332432532632732832933033133233333433533633733833934034134234334434534634734834935035135235335435535635735835936036136236336436536636736836937037137237337437537637737837938038138238338438538638738838939039139239339439539639739839940040140240340440540640740840941041141241341441541641741841942042142242342442542642742842943043143243343443543643743843944044144244344444544644744844945045145245345445545645745845946046146246346446546646746846947047147247347447547647747847948048148248348448548648748848949049149249349449549649749849950050150250350450550650750850951051151251351451551651751851952052152252352452552652752852953053153253353453553653753853954054154254354454554654754854955055155255355455555655755855956056156256356456556656756856957057157257357457557657757857958058158258358458558658758858959059159259359459559659759859960060160260360460560660760860961061161261361461561661761861962062162262362462562662762862963063163263363463563663763863964064164264364464564664764864965065165265365465565665765865966066166266366466566666766866967067167267367467567667767867968068168268368468568668768868969069169269369469569669769869970070170270370470570670770870971071171271371471571671771871972072172272372472572672772872973073173273373473573673773873974074174274374474574674774874975075175275375475575675775875976076176276376476576676776876977077177277377477577677777877978078178278378478578678778878979079179279379479579679779879980080180280380480580680780880981081181281381481581681781881982082182282382482582682782882983083183283383483583683783883984084184284384484584684784884985085185285385485585685785885986086186286386486586686786886987087187287387487587687787887988088188288388488588688788888989089189289389489589689789889990090190290390490590690790890991091191291391491591691791891992092192292392492592692792892993093193293393493593693793893994094194294394494594694794894995095195295395495595695795895996096196296396496596696796896997097197297397497597697797897998098198298398498598698798898999099199299399499599699799899910001001100210031004100510061007100810091010101110121013101410151016101710181019102010211022102310241025102610271028102910301031103210331034103510361037103810391040104110421043104410451046104710481049105010511052105310541055105610571058105910601061106210631064106510661067106810691070107110721073107410751076107710781079108010811082108310841085108610871088
  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.RangeMap
  595. Agda.Utils.SemiRing
  596. Agda.Utils.Semigroup
  597. Agda.Utils.Singleton
  598. Agda.Utils.Size
  599. Agda.Utils.SmallSet
  600. Agda.Utils.String
  601. Agda.Utils.Suffix
  602. Agda.Utils.Three
  603. Agda.Utils.Time
  604. Agda.Utils.Trie
  605. Agda.Utils.Tuple
  606. Agda.Utils.TypeLevel
  607. Agda.Utils.TypeLits
  608. Agda.Utils.Update
  609. Agda.Utils.VarSet
  610. Agda.Utils.Warshall
  611. Agda.Utils.WithDefault
  612. Agda.Utils.Zipper
  613. Agda.Version
  614. Agda.VersionCommit
  615. other-modules: Paths_Agda
  616. Agda.Interaction.Highlighting.Dot.Backend
  617. Agda.Interaction.Highlighting.Dot.Base
  618. Agda.Interaction.Highlighting.HTML.Backend
  619. Agda.Interaction.Highlighting.HTML.Base
  620. Agda.Interaction.Highlighting.LaTeX.Backend
  621. Agda.Interaction.Highlighting.LaTeX.Base
  622. Agda.Interaction.Options.Base
  623. Agda.Interaction.Options.HasOptions
  624. Agda.Utils.CallStack.Base
  625. Agda.Utils.CallStack.Pretty
  626. if flag(optimise-heavily)
  627. ghc-options: -fexpose-all-unfoldings
  628. -fspecialise-aggressively
  629. -- NOTE: If adding flags, also add to `.ghci-8.0`
  630. if impl(ghc <= 8.0.2)
  631. ghc-options: -fprint-potential-instances
  632. -- Initially, we disable all the warnings.
  633. -w
  634. -Werror
  635. -- This option must be the first one after disabling the
  636. -- warnings. See Issue #2094.
  637. -Wunrecognised-warning-flags
  638. -Wdeprecated-flags
  639. -Wderiving-typeable
  640. -Wdodgy-exports
  641. -Wdodgy-foreign-imports
  642. -Wdodgy-imports
  643. -Wduplicate-exports
  644. -Wempty-enumerations
  645. -Widentities
  646. -Wincomplete-patterns
  647. -Winline-rule-shadowing
  648. -Wmissing-fields
  649. -Wmissing-methods
  650. -Wmissing-pattern-synonym-signatures
  651. -Wmissing-signatures
  652. -Wnoncanonical-monad-instances
  653. -Wnoncanonical-monoid-instances
  654. -Woverflowed-literals
  655. -Woverlapping-patterns
  656. -Wsemigroup
  657. -Wtabs
  658. -Wtyped-holes
  659. -Wunrecognised-pragmas
  660. -Wunticked-promoted-constructors
  661. -Wunused-do-bind
  662. -Wunused-foralls
  663. -Wwarnings-deprecations
  664. -Wwrong-do-bind
  665. else
  666. ghc-options: -fprint-potential-instances
  667. -Werror=unrecognised-warning-flags
  668. -Werror=deprecated-flags
  669. -Werror=deriving-typeable
  670. -Werror=dodgy-exports
  671. -Werror=dodgy-foreign-imports
  672. -Werror=dodgy-imports
  673. -Werror=duplicate-exports
  674. -Werror=empty-enumerations
  675. -Werror=identities
  676. -Werror=incomplete-patterns
  677. -Werror=inline-rule-shadowing
  678. -Werror=missing-fields
  679. -Werror=missing-methods
  680. -Werror=missing-pattern-synonym-signatures
  681. -Werror=missing-signatures
  682. -Werror=noncanonical-monad-instances
  683. -Werror=noncanonical-monoid-instances
  684. -Werror=overflowed-literals
  685. -Werror=overlapping-patterns
  686. -Werror=semigroup
  687. -Werror=tabs
  688. -Werror=typed-holes
  689. -Werror=unrecognised-pragmas
  690. -Werror=unticked-promoted-constructors
  691. -Werror=unused-do-bind
  692. -Werror=unused-foralls
  693. -Werror=warnings-deprecations
  694. -Werror=wrong-do-bind
  695. -- NOTE: If adding or removing flags, also change `.ghci-8.2`
  696. if impl(ghc >= 8.2)
  697. ghc-options: -Wcpp-undef
  698. -- ASR TODO (2017-07-23): `make haddock` fails when
  699. -- this flag is on.
  700. -- -Wmissing-home-modules
  701. -Werror=simplifiable-class-constraints
  702. -Werror=unbanged-strict-patterns
  703. -- NOTE: If adding or removing flags, also change `.ghci-8.6`
  704. if impl(ghc >= 8.6)
  705. ghc-options: -Werror=inaccessible-code
  706. -Werror=star-binder
  707. -Werror=star-is-type
  708. -- The following warning is an error in GHC >= 8.10.
  709. if impl(ghc >= 8.6) && impl(ghc < 8.10)
  710. ghc-options: -Werror=implicit-kind-vars
  711. -- NOTE: If adding or removing flags, also change `.ghci-8.8`
  712. if impl(ghc >= 8.8)
  713. ghc-options: -Werror=missed-extra-shared-lib
  714. -- NOTE: If adding or removing flags, also change `.ghci-8.10`
  715. if impl(ghc >= 8.10)
  716. ghc-options: -Werror=deriving-defaults
  717. -Werror=redundant-record-wildcards
  718. -Werror=unused-packages
  719. -Werror=unused-record-wildcards
  720. -- NOTE: If adding or removing flags, also change `.ghci-9.0`
  721. if impl(ghc >= 9.0)
  722. ghc-options: -Werror=invalid-haddock
  723. ghc-prof-options: -fprof-auto
  724. default-language: Haskell2010
  725. -- NOTE: If adding or removing default extensions, also change:
  726. -- .ghci-8.0
  727. -- .hlint.yaml
  728. -- This should also use the same extensions as the `test-suite` target below.
  729. default-extensions: BangPatterns
  730. , ConstraintKinds
  731. --L-T Chen (2019-07-15):
  732. -- Enabling DataKinds only locally makes the compile time
  733. -- slightly shorter, see PR #3920.
  734. --, DataKinds
  735. , DefaultSignatures
  736. , DeriveDataTypeable
  737. , DeriveFoldable
  738. , DeriveFunctor
  739. , DeriveGeneric
  740. , DeriveTraversable
  741. , ExistentialQuantification
  742. , FlexibleContexts
  743. , FlexibleInstances
  744. , FunctionalDependencies
  745. , GeneralizedNewtypeDeriving
  746. , InstanceSigs
  747. , LambdaCase
  748. , MultiParamTypeClasses
  749. , MultiWayIf
  750. , NamedFieldPuns
  751. , OverloadedStrings
  752. , PatternSynonyms
  753. , RankNTypes
  754. , RecordWildCards
  755. , ScopedTypeVariables
  756. , StandaloneDeriving
  757. , TupleSections
  758. , TypeFamilies
  759. , TypeSynonymInstances
  760. executable agda
  761. hs-source-dirs: src/main
  762. main-is: Main.hs
  763. build-depends: Agda
  764. -- A version range on Agda generates a warning with
  765. -- some versions of Cabal and GHC
  766. -- (e.g. cabal-install version 1.24.0.2 compiled
  767. -- using version 1.24.2.0 of the Cabal library and
  768. -- GHC 8.2.1 RC1).
  769. -- Nothing is used from the following package,
  770. -- except for the Prelude.
  771. , base
  772. default-language: Haskell2010
  773. -- If someone installs Agda with the setuid bit set, then the
  774. -- presence of +RTS may be a security problem (see GHC bug #3910).
  775. -- However, we sometimes recommend people to use +RTS to control
  776. -- Agda's memory usage, so we want this functionality enabled by
  777. -- default.
  778. -- The threaded RTS by default starts a major GC after a program has
  779. -- been idle for 0.3 s. This feature turned out to be annoying, so
  780. -- the idle GC is now by default turned off (-I0).
  781. ghc-options: -threaded -rtsopts
  782. "-with-rtsopts=-M3.5G -I0"
  783. executable agda-mode
  784. hs-source-dirs: src/agda-mode
  785. main-is: Main.hs
  786. other-modules: Paths_Agda
  787. build-depends: base >= 4.9.0.0 && < 4.17
  788. , directory >= 1.2.6.2 && < 1.4
  789. , filepath >= 1.4.1.0 && < 1.5
  790. , process >= 1.4.2.0 && < 1.7
  791. default-language: Haskell2010
  792. -- Cabal testsuite integration has some serious bugs, but we
  793. -- can still make it work. See also:
  794. -- https://github.com/haskell/cabal/issues/1938
  795. -- https://github.com/haskell/cabal/issues/2214
  796. -- https://github.com/haskell/cabal/issues/1953
  797. --
  798. -- This test suite should only be run using the Makefile.
  799. -- The Makefile sets up the required environment,
  800. -- executing the tests using cabal directly is almost
  801. -- guaranteed to fail. See also Issue 1490.
  802. test-suite agda-tests
  803. type: exitcode-stdio-1.0
  804. hs-source-dirs: test/
  805. main-is: Main.hs
  806. other-modules: Bugs.Tests
  807. , Compiler.Tests
  808. , Fail.Tests
  809. , Interactive.Tests
  810. , Internal.Compiler.MAlonzo.Encode
  811. , Internal.Helpers
  812. , Internal.Interaction.Highlighting.Precise
  813. , Internal.Interaction.Highlighting.Range
  814. , Internal.Interaction.Library
  815. , Internal.Interaction.Options
  816. , Internal.Syntax.Abstract.Name
  817. , Internal.Syntax.Common
  818. , Internal.Syntax.Concrete.Name
  819. , Internal.Syntax.Internal
  820. , Internal.Syntax.Parser.Parser
  821. , Internal.Syntax.Position
  822. , Internal.Termination.CallGraph
  823. , Internal.Termination.CallMatrix
  824. , Internal.Termination.Order
  825. , Internal.Termination.Semiring
  826. , Internal.Termination.SparseMatrix
  827. , Internal.Termination.Termination
  828. , Internal.Tests
  829. , Internal.TypeChecking
  830. , Internal.TypeChecking.Free
  831. , Internal.TypeChecking.Free.Lazy
  832. , Internal.TypeChecking.Generators
  833. , Internal.TypeChecking.Irrelevance
  834. , Internal.TypeChecking.Monad.Base
  835. , Internal.TypeChecking.Positivity
  836. , Internal.TypeChecking.Positivity.Occurrence
  837. , Internal.TypeChecking.Rules.LHS.Problem
  838. , Internal.TypeChecking.SizedTypes
  839. , Internal.TypeChecking.SizedTypes.Syntax
  840. , Internal.TypeChecking.SizedTypes.WarshallSolver
  841. , Internal.TypeChecking.Substitute
  842. , Internal.Utils.AssocList
  843. , Internal.Utils.Bag
  844. , Internal.Utils.BiMap
  845. , Internal.Utils.Cluster
  846. , Internal.Utils.Either
  847. , Internal.Utils.Favorites
  848. , Internal.Utils.FileName
  849. , Internal.Utils.Graph.AdjacencyMap.Unidirectional
  850. , Internal.Utils.IntSet
  851. , Internal.Utils.List
  852. , Internal.Utils.ListT
  853. , Internal.Utils.Maybe.Strict
  854. , Internal.Utils.Monoid
  855. , Internal.Utils.NonEmptyList
  856. , Internal.Utils.PartialOrd
  857. , Internal.Utils.Permutation
  858. , Internal.Utils.RangeMap
  859. , Internal.Utils.SmallSet
  860. , Internal.Utils.Three
  861. , Internal.Utils.Trie
  862. , Internal.Utils.Warshall
  863. , LaTeXAndHTML.Tests
  864. , LibSucceed.Tests
  865. , Succeed.Tests
  866. , UserManual.Tests
  867. , Utils
  868. -- Andreas, 2021-08-26, see https://github.com/haskell/cabal/issues/7577
  869. -- Since 'agda-tests' wants to call 'agda', we have to add it here,
  870. -- should we want to run 'cabal test'.
  871. build-tool-depends: Agda:agda
  872. build-depends: Agda
  873. , array
  874. , base
  875. , bytestring
  876. , containers
  877. , directory
  878. , filepath
  879. , filemanip >= 0.3.6.3 && < 0.4
  880. , mtl
  881. , process
  882. , process-extras >= 0.3.0 && < 0.3.4 || >= 0.4.1.3 && < 0.5 || >= 0.7.1 && < 0.8
  883. , QuickCheck >= 2.14.1 && < 2.15
  884. , regex-tdfa
  885. , strict >= 0.3.2 && < 0.5
  886. , tasty >= 1.1.0.4 && < 1.5
  887. , tasty-hunit >= 0.9.2 && < 0.11
  888. , tasty-quickcheck >= 0.9.2 && < 0.11
  889. -- tasty-silver 3.1.13 has option --ansi-tricks=false
  890. -- NB: tasty-silver 3.2 requires tasty >= 1.4
  891. -- tasty-silver < 3.3 does not work interactively under Windows
  892. , tasty-silver >= 3.1.13 && < 3.4
  893. , temporary >= 1.2.0.3 && < 1.4
  894. , text
  895. , unix-compat >= 0.4.3.1 && < 0.6
  896. , unordered-containers >= 0.2.5.0 && < 0.3
  897. , uri-encode
  898. -- Andreas (2021-10-11): tasty-silver < 3.3 does not work interactively under Windows
  899. if os(windows)
  900. build-depends: tasty-silver >= 3.3
  901. default-language: Haskell2010
  902. -- NOTE: If adding or removing default extensions, also change:
  903. -- .ghci-8.0
  904. -- .hlint.yaml
  905. -- This should also use the same extensions as the `library` target above.
  906. default-extensions: BangPatterns
  907. , ConstraintKinds
  908. --L-T Chen (2019-07-15):
  909. -- Enabling DataKinds only locally makes the compile time
  910. -- slightly shorter, see PR #3920.
  911. --, DataKinds
  912. , DefaultSignatures
  913. , DeriveDataTypeable
  914. , DeriveFoldable
  915. , DeriveFunctor
  916. , DeriveGeneric
  917. , DeriveTraversable
  918. , ExistentialQuantification
  919. , FlexibleContexts
  920. , FlexibleInstances
  921. , FunctionalDependencies
  922. , GeneralizedNewtypeDeriving
  923. , InstanceSigs
  924. , LambdaCase
  925. , MultiParamTypeClasses
  926. , MultiWayIf
  927. , NamedFieldPuns
  928. , OverloadedStrings
  929. , PatternSynonyms
  930. , RankNTypes
  931. , RecordWildCards
  932. , ScopedTypeVariables
  933. , StandaloneDeriving
  934. , TupleSections
  935. , TypeFamilies
  936. , TypeSynonymInstances
  937. if flag(optimise-heavily)
  938. ghc-options: -fexpose-all-unfoldings
  939. -fspecialise-aggressively
  940. -- NOTE: If adding or removing flags, also change `.ghci-8.0`
  941. if impl(ghc <= 8.0.2)
  942. ghc-options: -threaded
  943. -- Initially, we disable all the warnings.
  944. -w
  945. -Werror
  946. -- This option must be the first one after disabling the
  947. -- warnings. See Issue #2094.
  948. -Wunrecognised-warning-flags
  949. -Wdeprecated-flags
  950. -Wderiving-typeable
  951. -Wdodgy-exports
  952. -Wdodgy-foreign-imports
  953. -Wdodgy-imports
  954. -Wduplicate-exports
  955. -Wempty-enumerations
  956. -Widentities
  957. -Wincomplete-patterns
  958. -Winline-rule-shadowing
  959. -Wmissing-fields
  960. -Wmissing-methods
  961. -Wmissing-pattern-synonym-signatures
  962. -Wmissing-signatures
  963. -Wnoncanonical-monad-instances
  964. -Wnoncanonical-monoid-instances
  965. -Woverflowed-literals
  966. -Woverlapping-patterns
  967. -Wsemigroup
  968. -Wtabs
  969. -Wtyped-holes
  970. -Wunrecognised-pragmas
  971. -Wunticked-promoted-constructors
  972. -Wunused-do-bind
  973. -Wunused-foralls
  974. -Wwarnings-deprecations
  975. -Wwrong-do-bind
  976. else
  977. ghc-options: -threaded
  978. -Werror=unrecognised-warning-flags
  979. -Werror=deprecated-flags
  980. -Werror=deriving-typeable
  981. -Werror=dodgy-exports
  982. -Werror=dodgy-foreign-imports
  983. -Werror=dodgy-imports
  984. -Werror=duplicate-exports
  985. -Werror=empty-enumerations
  986. -Werror=identities
  987. -Werror=incomplete-patterns
  988. -Werror=inline-rule-shadowing
  989. -Werror=missing-fields
  990. -Werror=missing-methods
  991. -Werror=missing-pattern-synonym-signatures
  992. -Werror=missing-signatures
  993. -Werror=noncanonical-monad-instances
  994. -Werror=noncanonical-monoid-instances
  995. -Werror=overflowed-literals
  996. -Werror=overlapping-patterns
  997. -Werror=semigroup
  998. -Werror=tabs
  999. -Werror=typed-holes
  1000. -Werror=unrecognised-pragmas
  1001. -Werror=unticked-promoted-constructors
  1002. -Werror=unused-do-bind
  1003. -Werror=unused-foralls
  1004. -Werror=warnings-deprecations
  1005. -Werror=wrong-do-bind
  1006. -- ASR (2017-04-11). TODO: Using -Werror=missing-home-modules generates an
  1007. -- error.
  1008. -- NOTE: If adding or removing flags, also change `.ghci-8.2`
  1009. if impl(ghc >= 8.2)
  1010. ghc-options: -Werror=cpp-undef
  1011. -Werror=simplifiable-class-constraints
  1012. -Werror=unbanged-strict-patterns
  1013. -- NOTE: If adding or removing flags, also change `.ghci-8.6`
  1014. if impl(ghc >= 8.6)
  1015. ghc-options: -Werror=inaccessible-code
  1016. -Werror=star-binder
  1017. -Werror=star-is-type
  1018. -- The following warning is an error in GHC >= 8.10.
  1019. if impl(ghc >= 8.6) && impl(ghc < 8.10)
  1020. ghc-options: -Werror=implicit-kind-vars
  1021. -- NOTE: If adding or removing flags, also change `.ghci-8.8`
  1022. if impl(ghc >= 8.8)
  1023. ghc-options: -Werror=missed-extra-shared-lib
  1024. -- NOTE: If adding or removing flags, also change `.ghci-8.10`
  1025. if impl(ghc >= 8.10)
  1026. ghc-options: -Werror=deriving-defaults
  1027. -Werror=redundant-record-wildcards
  1028. -Werror=unused-packages
  1029. -Werror=unused-record-wildcards
  1030. -- NOTE: If adding or removing flags, also change `.ghci-9.0`
  1031. if impl(ghc >= 9.0)
  1032. ghc-options: -Werror=compat-unqualified-imports
  1033. -Werror=invalid-haddock