Skip to content

Commit aef3643

Browse files
HeinrichApfelmusomelkonian
authored andcommitted
Rename Set to Type in tests
1 parent e0376a5 commit aef3643

File tree

88 files changed

+219
-190
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

88 files changed

+219
-190
lines changed

test/BangPatterns.agda

+2-2
Original file line numberDiff line numberDiff line change
@@ -19,13 +19,13 @@ foldl'' f (! x0) (x ∷ xs) = foldl'' f (! f x0 x) xs
1919

2020
{-# COMPILE AGDA2HS foldl'' #-}
2121

22-
data LazyMaybe (a : Set ℓ) : Setwhere
22+
data LazyMaybe (a : Type ℓ) : Typewhere
2323
LazyNothing : LazyMaybe a
2424
LazyJust : a LazyMaybe a
2525

2626
{-# COMPILE AGDA2HS LazyMaybe #-}
2727

28-
data StrictMaybe (a : Set ℓ) : Setwhere
28+
data StrictMaybe (a : Type ℓ) : Typewhere
2929
StrictNothing : StrictMaybe a
3030
StrictJust : Strict a StrictMaybe a
3131

test/CanonicalInstance.agda

+2-2
Original file line numberDiff line numberDiff line change
@@ -4,14 +4,14 @@ module _ where
44

55
open import Haskell.Prelude
66

7-
record ClassA (a : Set) : Set where
7+
record ClassA (a : Type) : Type where
88
field
99
myA : a
1010

1111
open ClassA ⦃ ... ⦄ public
1212
{-# COMPILE AGDA2HS ClassA class #-}
1313

14-
record ClassB (b : Set) : Set where
14+
record ClassB (b : Type) : Type where
1515
field
1616
overlap ⦃ super ⦄ : ClassA b
1717
{-# COMPILE AGDA2HS ClassB class #-}

test/Coerce.agda

+2-2
Original file line numberDiff line numberDiff line change
@@ -1,9 +1,9 @@
11
open import Haskell.Prelude
22

3-
data A : Set where
3+
data A : Type where
44
MkA : Nat A
55

6-
data B : Set where
6+
data B : Type where
77
MkB : Nat B
88

99
postulate A≡B : A ≡ B

test/Coinduction.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ module Coinduction where
55
open import Haskell.Prelude
66
open import Haskell.Prim.Thunk
77

8-
data Colist (a : Set) (@0 i : Size) : Set where
8+
data Colist (a : Type) (@0 i : Size) : Type where
99
Nil : Colist a i
1010
Cons : a -> Thunk (Colist a) i -> Colist a i
1111

test/ConstrainedInstance.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,7 @@
11

22
open import Haskell.Prelude
33

4-
data D (a : Set) : Set where
4+
data D (a : Type) : Type where
55
C : a D a
66
{-# COMPILE AGDA2HS D #-}
77

test/Cubical/StreamFusion.agda

+1-2
Original file line numberDiff line numberDiff line change
@@ -2,15 +2,14 @@ module Cubical.StreamFusion where
22

33
open import Haskell.Prelude
44

5-
open import Agda.Primitive
65
open import Agda.Primitive.Cubical
76
open import Agda.Builtin.Equality
87
open import Agda.Builtin.Size
98

109
variable
1110
@0 i : Size
1211

13-
record Stream (a : Set) (@0 i : Size) : Set where
12+
record Stream (a : Type) (@0 i : Size) : Type where
1413
pattern; inductive; constructor _:>_
1514
field
1615
shead : a

test/CustomTuples.agda

+4-4
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
open import Haskell.Prelude
22

3-
record Σ (a : Set) (b : @0 a Set) : Set where
3+
record Σ (a : Type) (b : @0 a Type) : Type where
44
constructor _,_
55
field
66
fst : a
@@ -13,7 +13,7 @@ test xy = fst xy + snd xy
1313

1414
{-# COMPILE AGDA2HS test #-}
1515

16-
record Stuff (a : Set) : Set where
16+
record Stuff (a : Type) : Type where
1717
no-eta-equality; pattern
1818
constructor stuff
1919
field
@@ -38,7 +38,7 @@ section = stuff 42
3838

3939
{-# COMPILE AGDA2HS section #-}
4040

41-
record NoStuff : Set where
41+
record NoStuff : Type where
4242
no-eta-equality; pattern
4343
constructor dontlook
4444

@@ -50,7 +50,7 @@ bar dontlook = dontlook
5050
{-# COMPILE AGDA2HS bar #-}
5151

5252
-- This is legal, basically the same as an unboxed record.
53-
record Legal (a : Set) : Set where
53+
record Legal (a : Type) : Type where
5454
constructor mkLegal
5555
field
5656
theA : a

test/Datatypes.agda

+2-2
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,7 @@
11

2-
open import Agda.Builtin.Bool
2+
open import Haskell.Prim using (Bool; Type)
33

4-
data Test : Set where
4+
data Test : Type where
55
CTest : Bool -> @0 {Bool} -> Test
66
{-# COMPILE AGDA2HS Test #-}
77

test/Default.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
open import Haskell.Prelude
22

3-
record HasDefault (a : Set) : Set where
3+
record HasDefault (a : Type) : Type where
44
field
55
theDefault : a
66
open HasDefault {{...}}

test/DefaultMethods.agda

+12-12
Original file line numberDiff line numberDiff line change
@@ -14,18 +14,18 @@ import Prelude hiding (Show, show, showsPrec, showList, Ord, (<), (>))
1414

1515
-- ** Ord
1616

17-
record Ord (a : Set) : Set where
17+
record Ord (a : Type) : Type where
1818
field
1919
_<_ _>_ : a a Bool
2020

21-
record Ord₁ (a : Set) : Set where
21+
record Ord₁ (a : Type) : Type where
2222
field
2323
_<_ : a a Bool
2424

2525
_>_ : a a Bool
2626
x > y = y < x
2727

28-
record Ord₂ (a : Set) : Set where
28+
record Ord₂ (a : Type) : Type where
2929
field
3030
_>_ : a a Bool
3131

@@ -46,7 +46,7 @@ instance
4646
OrdBool₀ ._>_ = Ord₁._>_ OB
4747
{-# COMPILE AGDA2HS OrdBool₀ #-}
4848

49-
data Bool1 : Set where
49+
data Bool1 : Type where
5050
Mk1 : Bool -> Bool1
5151
{-# COMPILE AGDA2HS Bool1 #-}
5252
instance
@@ -58,7 +58,7 @@ instance
5858
ord₁ .Ord₁._<_ (Mk1 True) _ = False
5959
{-# COMPILE AGDA2HS OrdBool₁ #-}
6060

61-
data Bool2 : Set where
61+
data Bool2 : Type where
6262
Mk2 : Bool -> Bool2
6363
{-# COMPILE AGDA2HS Bool2 #-}
6464
instance
@@ -70,7 +70,7 @@ instance
7070
(Mk2 True) <: _ = False
7171
{-# COMPILE AGDA2HS OrdBool₂ #-}
7272

73-
data Bool3 : Set where
73+
data Bool3 : Type where
7474
Mk3 : Bool -> Bool3
7575
{-# COMPILE AGDA2HS Bool3 #-}
7676
instance
@@ -82,7 +82,7 @@ instance
8282
(Mk3 True) <: _ = False
8383
{-# COMPILE AGDA2HS OrdBool₃ #-}
8484

85-
data Bool4 : Set where
85+
data Bool4 : Type where
8686
Mk4 : Bool -> Bool4
8787
{-# COMPILE AGDA2HS Bool4 #-}
8888
lift4 : (Bool Bool a) (Bool4 Bool4 a)
@@ -93,7 +93,7 @@ instance
9393
OrdBool₄ = record {Ord₁ (λ where .Ord₁._<_ lift4 (λ x y not x && y))}
9494
{-# COMPILE AGDA2HS OrdBool₄ #-}
9595

96-
data Bool5 : Set where
96+
data Bool5 : Type where
9797
Mk5 : Bool -> Bool5
9898
{-# COMPILE AGDA2HS Bool5 #-}
9999
instance
@@ -105,7 +105,7 @@ instance
105105
(Mk5 True) >: (Mk5 b) = not b
106106
{-# COMPILE AGDA2HS OrdBool₅ #-}
107107

108-
data Bool6 : Set where
108+
data Bool6 : Type where
109109
Mk6 : Bool -> Bool6
110110
{-# COMPILE AGDA2HS Bool6 #-}
111111
instance
@@ -131,13 +131,13 @@ defaultShowList shows (x ∷ xs)
131131
∘ showString "]"
132132
{-# COMPILE AGDA2HS defaultShowList #-}
133133

134-
record Show (a : Set) : Set where
134+
record Show (a : Type) : Type where
135135
field
136136
show : a String
137137
showsPrec : Int a ShowS
138138
showList : List a ShowS
139139

140-
record Show₁ (a : Set) : Set where
140+
record Show₁ (a : Type) : Type where
141141
field showsPrec : Int a ShowS
142142

143143
show : a String
@@ -146,7 +146,7 @@ record Show₁ (a : Set) : Set where
146146
showList : List a ShowS
147147
showList = defaultShowList (showsPrec 0)
148148

149-
record Show₂ (a : Set) : Set where
149+
record Show₂ (a : Type) : Type where
150150
field show : a String
151151

152152
showsPrec : Int a ShowS

test/Deriving.agda

+4-4
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
open import Haskell.Prelude
22

3-
data Planet : Set where
3+
data Planet : Type where
44
Mercury : Planet
55
Venus : Planet
66
Earth : Planet
@@ -36,7 +36,7 @@ postulate instance iPlanetShow : Show Planet
3636

3737
{-# COMPILE AGDA2HS iPlanetShow derive stock #-}
3838

39-
record Clazz (a : Set) : Set where
39+
record Clazz (a : Type) : Type where
4040
field
4141
foo : a Int
4242
bar : a Bool
@@ -49,7 +49,7 @@ postulate instance iPlanetClazz : Clazz Planet
4949

5050
{-# COMPILE AGDA2HS iPlanetClazz derive anyclass #-}
5151

52-
data Optional (a : Set) : Set where
52+
data Optional (a : Type) : Type where
5353
Of : a Optional a
5454
Empty : Optional a
5555

@@ -59,7 +59,7 @@ postulate instance iOptionalEq : ⦃ Eq a ⦄ → Eq (Optional a)
5959

6060
{-# COMPILE AGDA2HS iOptionalEq #-}
6161

62-
data Duo (a b : Set) : Set where
62+
data Duo (a b : Type) : Type where
6363
MkDuo : (a × b) Duo a b
6464

6565
{-# COMPILE AGDA2HS Duo newtype #-}

test/ErasedPatternLambda.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -2,7 +2,7 @@ open import Haskell.Prelude
22

33
Scope = List Bool
44

5-
data Telescope (@0 α : Scope) : @0 Scope Set where
5+
data Telescope (@0 α : Scope) : @0 Scope Type where
66
ExtendTel : {@0 x β} Bool Telescope (x ∷ α) β Telescope α (x ∷ β)
77
{-# COMPILE AGDA2HS Telescope #-}
88

test/ErasedTypeArguments.agda

+3-3
Original file line numberDiff line numberDiff line change
@@ -2,14 +2,14 @@
22
-- and in lambdas do get erased.
33
module ErasedTypeArguments where
44

5-
open import Agda.Primitive
5+
open import Agda.Primitive renaming (Set to Type)
66
open import Agda.Builtin.Unit
77
open import Agda.Builtin.Nat
88

99
-- A record type which has both members compiled,
1010
-- but the argument of the lambda is erased;
1111
-- so that it won't be dependent-typed after compilation.
12-
record Σ' {i j} (a : Set i) (b : @0 a -> Set j) : Set (i ⊔ j) where
12+
record Σ' {i j} (a : Type i) (b : @0 a -> Type j) : Type (i ⊔ j) where
1313
constructor _:^:_
1414
field
1515
proj₁ : a
@@ -26,6 +26,6 @@ test n = n :^: tt
2626

2727
-- Tests a type function that would be accepted anyway,
2828
-- but the argument is erased.
29-
data Id {i j} (@0 a : Set i) (f : @0 Set i -> Set j) : Set j where
29+
data Id {i j} (@0 a : Type i) (f : @0 Type i -> Type j) : Type j where
3030
MkId : f a -> Id a f
3131
{-# COMPILE AGDA2HS Id newtype #-}

test/Fail/Copatterns.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ module Fail.Copatterns where
44

55
open import Haskell.Prelude
66

7-
record R : Set where
7+
record R : Type where
88
field
99
foo : Bool
1010
open R public

test/Fail/DerivingParseFailure.agda

+3-1
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,8 @@
11
module Fail.DerivingParseFailure where
22

3-
record Example : Set where
3+
open import Haskell.Prim using (Type)
4+
5+
record Example : Type where
46
{-# COMPILE AGDA2HS Example deriving !& #-}
57
-- {-# COMPILE AGDA2HS Example deriving Show via Foo #-}
68
-- {-# COMPILE AGDA2HS Example deriving (Show, Eq, Ord) class #-}

test/Fail/ErasedRecordParameter.agda

+3-1
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,9 @@
11
-- c.f. Issue #145, this is the record variant
22
module Fail.ErasedRecordParameter where
33

4-
record Ok (@0 a : Set) : Set where
4+
open import Haskell.Prim using (Type)
5+
6+
record Ok (@0 a : Type) : Type where
57
constructor Thing
68
field unThing : a
79
open Ok public

test/Fail/ExplicitInstance.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ module Fail.ExplicitInstance where
33

44
open import Haskell.Prelude
55

6-
record HasDefault (a : Set) : Set where
6+
record HasDefault (a : Type) : Type where
77
field
88
theDefault : a
99
open HasDefault {{...}}

test/Fail/ExplicitInstance2.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ module Fail.ExplicitInstance2 where
33

44
open import Haskell.Prelude
55

6-
record HasDefault (a : Set) : Set where
6+
record HasDefault (a : Type) : Type where
77
field
88
theDefault : a
99
open HasDefault {{...}}

test/Fail/Issue113a.agda

+3-1
Original file line numberDiff line numberDiff line change
@@ -2,7 +2,9 @@
22

33
module Fail.Issue113a where
44

5-
record Loop : Set where
5+
open import Haskell.Prim using (Type)
6+
7+
record Loop : Type where
68
coinductive
79
field force : Loop
810
open Loop public

test/Fail/Issue113b.agda

+4-2
Original file line numberDiff line numberDiff line change
@@ -2,9 +2,11 @@
22

33
module Fail.Issue113b where
44

5-
postulate A : Set
5+
open import Haskell.Prim using (Type)
66

7-
record Loop : Set where
7+
postulate A : Type
8+
9+
record Loop : Type where
810
coinductive
911
field force : Loop
1012
open Loop public

test/Fail/Issue125.agda

+5-3
Original file line numberDiff line numberDiff line change
@@ -1,16 +1,18 @@
11
module Fail.Issue125 where
22

3-
data A (a : Set) : Set where
3+
open import Haskell.Prim using (Type)
4+
5+
data A (a : Type) : Type where
46
ACtr : a -> A a
57

68
{-# COMPILE AGDA2HS A #-}
79

8-
data B : Set where
10+
data B : Type where
911
ACtr : B
1012

1113
{-# COMPILE AGDA2HS B #-}
1214

13-
data C : Set where
15+
data C : Type where
1416
Ca : C
1517

1618
{-# COMPILE AGDA2HS C #-}

0 commit comments

Comments
 (0)