@@ -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 #-}
5252instance
@@ -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 #-}
6464instance
@@ -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 #-}
7676instance
@@ -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 #-}
8888lift4 : (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 #-}
9999instance
@@ -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 #-}
111111instance
@@ -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
0 commit comments