Skip to content

Commit 7eb3cc0

Browse files
gallaisMatthewDaggitt
authored andcommitted
[ fix #698 ] Make reflection module type check under --safe (#799)
* [ float ] bringing in the new agda features * [ name ] with safe decidable equality * [ meta ] with safe decidable equality * [ reflection ] safe and compatible with --without-K * [ literal ] moved to their own file * [ reflection ] more deprecations * [ cleanup ] import list of Reflection * [ reflection ] extracting Argument, Pattern Also cleanup, deprecation, new unArg-dec magic. * [ fix ] removing Reflection from the list of unsafe modules * [ changelog ] list new modules * [ deprecation ] of arg-info injectivity proofs * [ abstraction ] taken to its own module * [ build ] removing fake unsafe files, cleaning up GenerateEverything * [ refactor ] introducing DecidableEquality * [ re #803 ] 'gradual' decidable equality combinator for list * [ reflection ] putting Term in its own module Some cleaning up still needed. However I am stuck on a refactoring. * [ fix ] forgot to add Reflection.Term + Additional cleanup * [ fix ] no need to deprecate *private* definitions! * [ deprecated ] functions moved to Reflection.Term * [ reflection ] moving Definition to Reflection.Definition * [ typo ] * [ cosmetic ] more uses of DecidableEquality * [ changelog ] new modules
1 parent b067409 commit 7eb3cc0

24 files changed

+1359
-692
lines changed

.travis.yml

+1-1
Original file line numberDiff line numberDiff line change
@@ -30,7 +30,7 @@ install:
3030
# installing the dev version of Agda
3131
- git clone https://github.com/agda/agda
3232
- cd agda
33-
- git checkout b57260d0ceb1de4a5edc323d8ec2361904b5066e
33+
- git checkout 39c273eb6eb3ab68c23b0de7a19eaadd84f0e5fb
3434
# checking whether .ghc is still valid
3535
- cabal install alex happy
3636
- cabal install --only-dependencies --dry -v > $HOME/installplan.txt

CHANGELOG.md

+25-4
Original file line numberDiff line numberDiff line change
@@ -66,6 +66,9 @@ New modules
6666
Data.AVL.NonEmpty
6767
Data.AVL.NonEmpty.Propositional
6868
69+
Data.Float.Base
70+
Data.Float.Properties
71+
6972
Data.List.Membership.Propositional.Properties.WithK
7073
7174
Data.List.Relation.Binary.Disjoint.Propositional
@@ -101,6 +104,18 @@ New modules
101104
Data.Word.Base
102105
Data.Word.Properties
103106
107+
Reflection.Abstraction
108+
Reflection.Argument
109+
Reflection.Argument.Information
110+
Reflection.Argument.Relevance
111+
Reflection.Argument.Visibility
112+
Reflection.Definition
113+
Reflection.Literal
114+
Reflection.Meta
115+
Reflection.Name
116+
Reflection.Pattern
117+
Reflection.Term
118+
104119
Relation.Binary.Construct.Closure.Equivalence.Properties
105120
Relation.Binary.Rewriting
106121
@@ -218,8 +233,8 @@ been attached to all deprecated names.
218233
favour of `` and `tt` from `Data.Unit`, as it turns out that the latter
219234
have been automatically mapped to the Haskell equivalent for quite some time.
220235

221-
* The module `Data.Word.Unsafe` has been deprecated as there are no
222-
longer any unsafe operations.
236+
* The modules `Data.Word.Unsafe` and `Data.Float.Unsafe` have been removed
237+
as there are no longer any unsafe operations.
223238

224239
* Renamed a few `-identity` lemmas in `Codata.Stream.Properties` as they were
225240
proving two streams bisimilar rather than propositionally equal.
@@ -355,6 +370,9 @@ Other minor additions
355370
toNatDigits : (base : ℕ) {base≤16 : True (1 ≤? base)} → ℕ → List ℕ
356371
```
357372

373+
* Decidable equality over floating point numbers has been made safe and
374+
so `_≟_` has been moved from `Data.Float.Unsafe` to `Data.Float.Properties`.
375+
358376
* Added new pattern synonyms to `Data.Integer`:
359377
```agda
360378
pattern +0 = + 0
@@ -397,6 +415,8 @@ Other minor additions
397415
foldr-preservesᵇ : (P x → P y → P (f x y)) → P e → All P xs → P (foldr f e xs)
398416
foldr-preservesʳ : (P y → P (f x y)) → P e → P (foldr f e xs)
399417
foldr-preservesᵒ : (P x ⊎ P y → P (f x y)) → P e ⊎ Any P xs → P (foldr f e xs)
418+
419+
∷-dec : Dec (x ≡ y) → Dec (xs ≡ ys) → Dec (x List.∷ xs ≡ y ∷ ys)
400420
```
401421

402422
* Defined a new utility in `Data.List.Relation.Binary.Permutation.Inductive.Properties`:
@@ -637,8 +657,9 @@ Other minor additions
637657

638658
* Added new definitions in `Relation.Binary.Core`:
639659
```agda
640-
Universal _∼_ = ∀ x y → x ∼ y
641-
Recomputable _~_ = ∀ {x y} → .(x ~ y) → x ~ y
660+
Universal _∼_ = ∀ x y → x ∼ y
661+
Recomputable _~_ = ∀ {x y} → .(x ~ y) → x ~ y
662+
DecidableEquality A = Decidable {A = A} _≡_
642663
```
643664

644665
* Added new proof to `Relation.Binary.Consequences`:

GenerateEverything.hs

+33-47
Original file line numberDiff line numberDiff line change
@@ -1,9 +1,11 @@
11
{-# LANGUAGE PatternGuards #-}
22

33
import Control.Applicative
4+
import Control.Monad
45

56
import qualified Data.List as List
67

8+
import System.Directory
79
import System.Environment
810
import System.Exit
911
import System.FilePath
@@ -21,7 +23,7 @@ srcDir = "src"
2123
-- | Checks whether a module is declared (un)safe
2224

2325
unsafeModules :: [FilePath]
24-
unsafeModules = map toAgdaFilePath
26+
unsafeModules = map modToFile
2527
[ "Codata.Musical.Cofin"
2628
, "Codata.Musical.Colist"
2729
, "Codata.Musical.Colist.Infinite-merge"
@@ -30,37 +32,37 @@ unsafeModules = map toAgdaFilePath
3032
, "Codata.Musical.Covec"
3133
, "Codata.Musical.M"
3234
, "Codata.Musical.Stream"
33-
, "Data.Char.Unsafe"
34-
, "Data.Float.Unsafe"
35-
, "Data.Nat.Unsafe"
36-
, "Data.Nat.DivMod.Unsafe"
37-
, "Data.String.Unsafe"
38-
, "Data.Word.Unsafe"
3935
, "Debug.Trace"
4036
, "Foreign.Haskell"
4137
, "IO"
4238
, "IO.Primitive"
43-
, "Reflection"
4439
, "Relation.Binary.PropositionalEquality.TrustMe"
4540
] where
4641

47-
toAgdaFilePath :: String -> FilePath
48-
toAgdaFilePath name = concat
49-
[ "src/"
50-
, map (\ c -> if c == '.' then '/' else c) name
51-
, ".agda"
52-
]
53-
5442
isUnsafeModule :: FilePath -> Bool
55-
isUnsafeModule =
56-
-- GA 2019-02-24: it is crucial to use an anonymous lambda
57-
-- here so that `unsafeModules` is shared between all calls
58-
-- to `isUnsafeModule`.
59-
\ fp -> unqualifiedModuleName fp == "Unsafe"
60-
|| fp `elem` unsafeModules
43+
isUnsafeModule fp =
44+
unqualifiedModuleName fp == "Unsafe"
45+
|| fp `elem` unsafeModules
6146

6247
-- | Checks whether a module is declared as using K
6348

49+
withKModules :: [FilePath]
50+
withKModules = map modToFile
51+
[ "Axiom.Extensionality.Heterogeneous"
52+
, "Data.Star.BoundedVec"
53+
, "Data.Star.Decoration"
54+
, "Data.Star.Environment"
55+
, "Data.Star.Fin"
56+
, "Data.Star.Pointer"
57+
, "Data.Star.Vec"
58+
, "Data.String.Unsafe"
59+
, "Relation.Binary.HeterogeneousEquality"
60+
, "Relation.Binary.HeterogeneousEquality.Core"
61+
, "Relation.Binary.HeterogeneousEquality.Quotients.Examples"
62+
, "Relation.Binary.HeterogeneousEquality.Quotients"
63+
, "Relation.Binary.PropositionalEquality.TrustMe"
64+
]
65+
6466
isWithKModule :: FilePath -> Bool
6567
isWithKModule =
6668
-- GA 2019-02-24: it is crucial to use an anonymous lambda
@@ -69,31 +71,6 @@ isWithKModule =
6971
\ fp -> unqualifiedModuleName fp == "WithK"
7072
|| fp `elem` withKModules
7173

72-
where
73-
74-
withKModules :: [FilePath]
75-
withKModules = map modToFile
76-
[ "Axiom.Extensionality.Heterogeneous"
77-
, "Data.Char.Unsafe"
78-
, "Data.Float.Unsafe"
79-
, "Data.Nat.Unsafe"
80-
, "Data.Nat.DivMod.Unsafe"
81-
, "Data.Star.BoundedVec"
82-
, "Data.Star.Decoration"
83-
, "Data.Star.Environment"
84-
, "Data.Star.Fin"
85-
, "Data.Star.Pointer"
86-
, "Data.Star.Vec"
87-
, "Data.String.Unsafe"
88-
, "Data.Word.Unsafe"
89-
, "Reflection"
90-
, "Relation.Binary.HeterogeneousEquality"
91-
, "Relation.Binary.HeterogeneousEquality.Core"
92-
, "Relation.Binary.HeterogeneousEquality.Quotients.Examples"
93-
, "Relation.Binary.HeterogeneousEquality.Quotients"
94-
, "Relation.Binary.PropositionalEquality.TrustMe"
95-
]
96-
9774
unqualifiedModuleName :: FilePath -> String
9875
unqualifiedModuleName = dropExtension . takeFileName
9976

@@ -104,7 +81,6 @@ isLibraryModule f =
10481
takeExtension f `elem` [".agda", ".lagda"]
10582
&& unqualifiedModuleName f /= "Core"
10683

107-
10884
---------------------------------------------------------------------------
10985
-- Analysing library files
11086

@@ -209,6 +185,13 @@ analyse fp = do
209185
, status = classify fp hd ls
210186
}
211187

188+
checkFilePaths :: String -> [FilePath] -> IO ()
189+
checkFilePaths cat fps = forM_ fps $ \ fp -> do
190+
b <- doesFileExist fp
191+
if b
192+
then pure ()
193+
else error $ fp ++ " is listed as " ++ cat ++ " but does not exist."
194+
212195
---------------------------------------------------------------------------
213196
-- Collecting all non-Core library files, analysing them and generating
214197
-- 4 files:
@@ -223,6 +206,9 @@ main = do
223206
[] -> return ()
224207
_ -> hPutStr stderr usage >> exitFailure
225208

209+
checkFilePaths "unsafe" unsafeModules
210+
checkFilePaths "using K" withKModules
211+
226212
header <- readFileUTF8 headerFile
227213
modules <- filter isLibraryModule . List.sort <$>
228214
find always

lib.cabal

+1
Original file line numberDiff line numberDiff line change
@@ -14,6 +14,7 @@ executable GenerateEverything
1414
main-is: GenerateEverything.hs
1515
default-language: Haskell2010
1616
build-depends: base >= 4.9.0.0 && < 4.13
17+
, directory >= 1.0.0.0 && < 1.4
1718
, filemanip >= 0.3.6.2 && < 0.4
1819
, filepath >= 1.4.1.0 && < 1.5
1920

src/Data/Float.agda

+4-16
Original file line numberDiff line numberDiff line change
@@ -1,27 +1,15 @@
11
------------------------------------------------------------------------
22
-- The Agda standard library
33
--
4-
-- Floats
4+
-- Floating point numbers
55
------------------------------------------------------------------------
66

77
{-# OPTIONS --without-K --safe #-}
88

99
module Data.Float where
1010

11-
open import Data.String.Base using (String)
12-
13-
------------------------------------------------------------------------
14-
-- Re-export built-ins publically
15-
16-
open import Agda.Builtin.Float public
17-
using
18-
( Float
19-
; primFloatEquality
20-
; primShowFloat
21-
)
22-
2311
------------------------------------------------------------------------
24-
-- Operations
12+
-- Re-export base definitions and decidability of equality
2513

26-
show : Float String
27-
show = primShowFloat
14+
open import Data.Float.Base public
15+
open import Data.Float.Properties using (_≈?_; _<?_; _≟_; _==_) public

src/Data/Float/Base.agda

+55
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,55 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- Floats: basic types and operations
5+
------------------------------------------------------------------------
6+
7+
{-# OPTIONS --without-K --safe #-}
8+
9+
module Data.Float.Base where
10+
11+
open import Relation.Binary.Core using (Rel)
12+
import Data.Word.Base as Word
13+
open import Function using (_on_)
14+
open import Agda.Builtin.Equality
15+
16+
------------------------------------------------------------------------
17+
-- Re-export built-ins publically
18+
19+
open import Agda.Builtin.Float public
20+
using (Float)
21+
renaming
22+
-- Relations
23+
( primFloatEquality to _≡ᵇ_
24+
; primFloatLess to _≤ᵇ_
25+
; primFloatNumericalEquality to _≈ᵇ_
26+
; primFloatNumericalLess to _≲ᵇ_
27+
-- Conversions
28+
; primShowFloat to show
29+
; primFloatToWord64 to toWord
30+
; primNatToFloat to fromℕ
31+
-- Operations
32+
; primFloatPlus to _+_
33+
; primFloatMinus to _-_
34+
; primFloatTimes to _*_
35+
; primFloatNegate to -_
36+
; primFloatDiv to _÷_
37+
; primFloatSqrt to sqrt
38+
; primRound to round
39+
; primFloor to ⌊_⌋
40+
; primCeiling to ⌈_⌉
41+
; primExp to e^_
42+
; primLog to log
43+
; primSin to sin
44+
; primCos to cos
45+
; primTan to tan
46+
; primASin to asin
47+
; primACos to acos
48+
; primATan to atan
49+
)
50+
51+
_≈_ : Rel Float _
52+
_≈_ = Word._≈_ on toWord
53+
54+
_<_ : Rel Float _
55+
_<_ = Word._<_ on toWord

0 commit comments

Comments
 (0)