@@ -43,13 +43,15 @@ record Setoid c ℓ : Set (suc (c ⊔ ℓ)) where
4343 isEquivalence : IsEquivalence _≈_
4444
4545 open IsEquivalence isEquivalence public
46+ using (refl; reflexive; isPartialEquivalence)
4647
4748 partialSetoid : PartialSetoid c ℓ
4849 partialSetoid = record
4950 { isPartialEquivalence = isPartialEquivalence
5051 }
5152
52- open PartialSetoid partialSetoid public using (_≉_)
53+ open PartialSetoid partialSetoid public
54+ hiding (Carrier; _≈_; isPartialEquivalence)
5355
5456
5557record DecSetoid c ℓ : Set (suc (c ⊔ ℓ)) where
@@ -60,14 +62,15 @@ record DecSetoid c ℓ : Set (suc (c ⊔ ℓ)) where
6062 isDecEquivalence : IsDecEquivalence _≈_
6163
6264 open IsDecEquivalence isDecEquivalence public
65+ using (_≟_; isEquivalence)
6366
6467 setoid : Setoid c ℓ
6568 setoid = record
6669 { isEquivalence = isEquivalence
6770 }
6871
69- open Setoid setoid public using (partialSetoid; _≉_)
70-
72+ open Setoid setoid public
73+ hiding (Carrier; _≈_; isEquivalence)
7174
7275------------------------------------------------------------------------
7376-- Preorders
@@ -99,6 +102,9 @@ record Preorder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
99102 infix 4 _≳_
100103 _≳_ = flip _≲_
101104
105+ infix 4 _⋧_
106+ _⋧_ = flip _⋦_
107+
102108 -- Deprecated.
103109 infix 4 _∼_
104110 _∼_ = _≲_
@@ -117,14 +123,15 @@ record TotalPreorder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
117123 isTotalPreorder : IsTotalPreorder _≈_ _≲_
118124
119125 open IsTotalPreorder isTotalPreorder public
120- hiding ( module Eq )
126+ using (total; isPreorder )
121127
122128 preorder : Preorder c ℓ₁ ℓ₂
123- preorder = record { isPreorder = isPreorder }
129+ preorder = record
130+ { isPreorder = isPreorder
131+ }
124132
125133 open Preorder preorder public
126- using (module Eq ; _≳_; _⋦_)
127-
134+ hiding (Carrier; _≈_; _≲_; isPreorder)
128135
129136------------------------------------------------------------------------
130137-- Partial orders
@@ -139,16 +146,21 @@ record Poset c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
139146 isPartialOrder : IsPartialOrder _≈_ _≤_
140147
141148 open IsPartialOrder isPartialOrder public
142- hiding ( module Eq )
149+ using (antisym; isPreorder )
143150
144151 preorder : Preorder c ℓ₁ ℓ₂
145152 preorder = record
146153 { isPreorder = isPreorder
147154 }
148155
149156 open Preorder preorder public
150- using (module Eq )
151- renaming (_⋦_ to _≰_)
157+ hiding (Carrier; _≈_; _≲_; isPreorder)
158+ renaming
159+ ( _⋦_ to _≰_; _≳_ to _≥_; _⋧_ to _≱_
160+ ; ≲-respˡ-≈ to ≤-respˡ-≈
161+ ; ≲-respʳ-≈ to ≤-respʳ-≈
162+ ; ≲-resp-≈ to ≤-resp-≈
163+ )
152164
153165
154166record DecPoset c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
@@ -159,17 +171,18 @@ record DecPoset c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
159171 _≤_ : Rel Carrier ℓ₂
160172 isDecPartialOrder : IsDecPartialOrder _≈_ _≤_
161173
162- private
163- module DPO = IsDecPartialOrder isDecPartialOrder
164- open DPO public hiding (module Eq )
174+ private module DPO = IsDecPartialOrder isDecPartialOrder
175+
176+ open DPO public
177+ using (_≟_; _≤?_; isPartialOrder)
165178
166179 poset : Poset c ℓ₁ ℓ₂
167180 poset = record
168181 { isPartialOrder = isPartialOrder
169182 }
170183
171184 open Poset poset public
172- using (preorder ; _≰_ )
185+ hiding (Carrier ; _≈_; _≤_; isPartialOrder; module Eq )
173186
174187 module Eq where
175188 decSetoid : DecSetoid c ℓ₁
@@ -203,6 +216,12 @@ record StrictPartialOrder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂))
203216 _≮_ : Rel Carrier _
204217 x ≮ y = ¬ (x < y)
205218
219+ infix 4 _>_
220+ _>_ = flip _<_
221+
222+ infix 4 _≯_
223+ _≯_ = flip _≮_
224+
206225
207226record DecStrictPartialOrder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
208227 infix 4 _≈_ _<_
@@ -212,17 +231,18 @@ record DecStrictPartialOrder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂
212231 _<_ : Rel Carrier ℓ₂
213232 isDecStrictPartialOrder : IsDecStrictPartialOrder _≈_ _<_
214233
215- private
216- module DSPO = IsDecStrictPartialOrder isDecStrictPartialOrder
217- open DSPO public hiding (module Eq )
234+ private module DSPO = IsDecStrictPartialOrder isDecStrictPartialOrder
235+
236+ open DSPO public
237+ using (_<?_; _≟_; isStrictPartialOrder)
218238
219239 strictPartialOrder : StrictPartialOrder c ℓ₁ ℓ₂
220240 strictPartialOrder = record
221241 { isStrictPartialOrder = isStrictPartialOrder
222242 }
223243
224244 open StrictPartialOrder strictPartialOrder public
225- using (_≮_ )
245+ hiding (Carrier; _≈_; _<_; isStrictPartialOrder; module Eq )
226246
227247 module Eq where
228248
@@ -247,15 +267,15 @@ record TotalOrder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
247267 isTotalOrder : IsTotalOrder _≈_ _≤_
248268
249269 open IsTotalOrder isTotalOrder public
250- hiding ( module Eq )
270+ using (total; isPartialOrder; isTotalPreorder )
251271
252272 poset : Poset c ℓ₁ ℓ₂
253273 poset = record
254274 { isPartialOrder = isPartialOrder
255275 }
256276
257277 open Poset poset public
258- using ( module Eq ; preorder ; _≰_ )
278+ hiding (Carrier; _≈_ ; _≤_; isPartialOrder )
259279
260280 totalPreorder : TotalPreorder c ℓ₁ ℓ₂
261281 totalPreorder = record
@@ -271,17 +291,18 @@ record DecTotalOrder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
271291 _≤_ : Rel Carrier ℓ₂
272292 isDecTotalOrder : IsDecTotalOrder _≈_ _≤_
273293
274- private
275- module DTO = IsDecTotalOrder isDecTotalOrder
276- open DTO public hiding (module Eq )
294+ private module DTO = IsDecTotalOrder isDecTotalOrder
295+
296+ open DTO public
297+ using (_≟_; _≤?_; isTotalOrder; isDecPartialOrder)
277298
278299 totalOrder : TotalOrder c ℓ₁ ℓ₂
279300 totalOrder = record
280301 { isTotalOrder = isTotalOrder
281302 }
282303
283304 open TotalOrder totalOrder public
284- using (poset; preorder ; _≰_ )
305+ hiding (Carrier; _≈_ ; _≤_; isTotalOrder; module Eq )
285306
286307 decPoset : DecPoset c ℓ₁ ℓ₂
287308 decPoset = record
@@ -306,25 +327,37 @@ record StrictTotalOrder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) wh
306327 isStrictTotalOrder : IsStrictTotalOrder _≈_ _<_
307328
308329 open IsStrictTotalOrder isStrictTotalOrder public
309- hiding (module Eq )
330+ using
331+ ( _≟_; _<?_; compare; isStrictPartialOrder
332+ ; isDecStrictPartialOrder; isDecEquivalence
333+ )
310334
311335 strictPartialOrder : StrictPartialOrder c ℓ₁ ℓ₂
312336 strictPartialOrder = record
313337 { isStrictPartialOrder = isStrictPartialOrder
314338 }
315339
316340 open StrictPartialOrder strictPartialOrder public
317- using (module Eq ; _≮_)
341+ hiding (Carrier; _≈_; _<_; isStrictPartialOrder; module Eq )
342+
343+ decStrictPartialOrder : DecStrictPartialOrder c ℓ₁ ℓ₂
344+ decStrictPartialOrder = record
345+ { isDecStrictPartialOrder = isDecStrictPartialOrder
346+ }
347+
348+ open DecStrictPartialOrder decStrictPartialOrder public
349+ using (module Eq )
318350
319351 decSetoid : DecSetoid c ℓ₁
320352 decSetoid = record
321- { isDecEquivalence = isDecEquivalence
353+ { isDecEquivalence = Eq. isDecEquivalence
322354 }
323355 {-# WARNING_ON_USAGE decSetoid
324356 "Warning: decSetoid was deprecated in v1.3.
325357 Please use Eq.decSetoid instead."
326358 #-}
327359
360+
328361record DenseLinearOrder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
329362 infix 4 _≈_ _<_
330363 field
@@ -342,6 +375,7 @@ record DenseLinearOrder c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) wh
342375 }
343376
344377 open StrictTotalOrder strictTotalOrder public
378+ hiding (Carrier; _≈_; _<_; isStrictTotalOrder)
345379
346380
347381------------------------------------------------------------------------
0 commit comments