@@ -14,18 +14,18 @@ import Prelude hiding (Show, show, showsPrec, showList, Ord, (<), (>))
14
14
15
15
-- ** Ord
16
16
17
- record Ord (a : Set ) : Set where
17
+ record Ord (a : Type ) : Type where
18
18
field
19
19
_<_ _>_ : a → a → Bool
20
20
21
- record Ord₁ (a : Set ) : Set where
21
+ record Ord₁ (a : Type ) : Type where
22
22
field
23
23
_<_ : a → a → Bool
24
24
25
25
_>_ : a → a → Bool
26
26
x > y = y < x
27
27
28
- record Ord₂ (a : Set ) : Set where
28
+ record Ord₂ (a : Type ) : Type where
29
29
field
30
30
_>_ : a → a → Bool
31
31
@@ -46,7 +46,7 @@ instance
46
46
OrdBool₀ ._>_ = Ord₁._>_ OB
47
47
{-# COMPILE AGDA2HS OrdBool₀ #-}
48
48
49
- data Bool1 : Set where
49
+ data Bool1 : Type where
50
50
Mk1 : Bool -> Bool1
51
51
{-# COMPILE AGDA2HS Bool1 #-}
52
52
instance
@@ -58,7 +58,7 @@ instance
58
58
ord₁ .Ord₁._<_ (Mk1 True) _ = False
59
59
{-# COMPILE AGDA2HS OrdBool₁ #-}
60
60
61
- data Bool2 : Set where
61
+ data Bool2 : Type where
62
62
Mk2 : Bool -> Bool2
63
63
{-# COMPILE AGDA2HS Bool2 #-}
64
64
instance
@@ -70,7 +70,7 @@ instance
70
70
(Mk2 True) <: _ = False
71
71
{-# COMPILE AGDA2HS OrdBool₂ #-}
72
72
73
- data Bool3 : Set where
73
+ data Bool3 : Type where
74
74
Mk3 : Bool -> Bool3
75
75
{-# COMPILE AGDA2HS Bool3 #-}
76
76
instance
@@ -82,7 +82,7 @@ instance
82
82
(Mk3 True) <: _ = False
83
83
{-# COMPILE AGDA2HS OrdBool₃ #-}
84
84
85
- data Bool4 : Set where
85
+ data Bool4 : Type where
86
86
Mk4 : Bool -> Bool4
87
87
{-# COMPILE AGDA2HS Bool4 #-}
88
88
lift4 : (Bool → Bool → a) → (Bool4 → Bool4 → a)
@@ -93,7 +93,7 @@ instance
93
93
OrdBool₄ = record {Ord₁ (λ where .Ord₁._<_ → lift4 (λ x y → not x && y))}
94
94
{-# COMPILE AGDA2HS OrdBool₄ #-}
95
95
96
- data Bool5 : Set where
96
+ data Bool5 : Type where
97
97
Mk5 : Bool -> Bool5
98
98
{-# COMPILE AGDA2HS Bool5 #-}
99
99
instance
@@ -105,7 +105,7 @@ instance
105
105
(Mk5 True) >: (Mk5 b) = not b
106
106
{-# COMPILE AGDA2HS OrdBool₅ #-}
107
107
108
- data Bool6 : Set where
108
+ data Bool6 : Type where
109
109
Mk6 : Bool -> Bool6
110
110
{-# COMPILE AGDA2HS Bool6 #-}
111
111
instance
@@ -131,13 +131,13 @@ defaultShowList shows (x ∷ xs)
131
131
∘ showString "]"
132
132
{-# COMPILE AGDA2HS defaultShowList #-}
133
133
134
- record Show (a : Set ) : Set where
134
+ record Show (a : Type ) : Type where
135
135
field
136
136
show : a → String
137
137
showsPrec : Int → a → ShowS
138
138
showList : List a → ShowS
139
139
140
- record Show₁ (a : Set ) : Set where
140
+ record Show₁ (a : Type ) : Type where
141
141
field showsPrec : Int → a → ShowS
142
142
143
143
show : a → String
@@ -146,7 +146,7 @@ record Show₁ (a : Set) : Set where
146
146
showList : List a → ShowS
147
147
showList = defaultShowList (showsPrec 0 )
148
148
149
- record Show₂ (a : Set ) : Set where
149
+ record Show₂ (a : Type ) : Type where
150
150
field show : a → String
151
151
152
152
showsPrec : Int → a → ShowS
0 commit comments