Skip to content

Commit 97b2a46

Browse files
Make names in NonStrict and Strict consistent
1 parent 2b67b08 commit 97b2a46

File tree

2 files changed

+13
-13
lines changed

2 files changed

+13
-13
lines changed

src/Data/Vec/Relation/Binary/Lex/NonStrict.agda

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -94,8 +94,8 @@ module _ {_≈_ : Rel A ℓ₁} {_≼_ : Rel A ℓ₂} where
9494
<-cmp ≈-sym _≟_ ≼-antisym ≼-total = Strict.<-cmp ≈-sym
9595
(Conv.<-trichotomous _ _ ≈-sym _≟_ ≼-antisym ≼-total)
9696

97-
<? : Decidable _≈_ Decidable _≼_ {m n} Decidable (_<_ {m} {n})
98-
<? _≟_ _≼?_ = Core.decidable (no id) _≟_
97+
<-dec : Decidable _≈_ Decidable _≼_ {m n} Decidable (_<_ {m} {n})
98+
<-dec _≟_ _≼?_ = Core.decidable (no id) _≟_
9999
(Conv.<-decidable _ _ _≟_ _≼?_)
100100

101101
------------------------------------------------------------------------
@@ -180,9 +180,9 @@ module _ {_≈_ : Rel A ℓ₁} {_≼_ : Rel A ℓ₂} where
180180
≤-total ≈-sym _≟_ ≼-antisym ≼-total = Strict.≤-total ≈-sym
181181
(Conv.<-trichotomous _ _ ≈-sym _≟_ ≼-antisym ≼-total)
182182

183-
? : Decidable _≈_ Decidable _≼_
184-
{m n} Decidable (_≤_ {m} {n})
185-
? _≟_ _≼?_ = Core.decidable (yes tt) _≟_
183+
-dec : Decidable _≈_ Decidable _≼_
184+
{m n} Decidable (_≤_ {m} {n})
185+
-dec _≟_ _≼?_ = Core.decidable (yes tt) _≟_
186186
(Conv.<-decidable _ _ _≟_ _≼?_)
187187

188188
≤-resp₂ : IsEquivalence _≈_ _≼_ Respects₂ _≈_

src/Data/Vec/Relation/Binary/Lex/Strict.agda

Lines changed: 8 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -177,9 +177,9 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
177177
{n} Antisymmetric (_≋_ {n} {n}) _≤_
178178
≤-antisym = Core.antisym
179179

180-
≤-respects: IsPartialEquivalence _≈_ _≺_ Respects₂ _≈_
181-
{n} _Respects₂_ (_≤_ {n} {n}) _≋_
182-
≤-respects= Core.respects₂
180+
≤-resp: IsPartialEquivalence _≈_ _≺_ Respects₂ _≈_
181+
{n} _Respects₂_ (_≤_ {n} {n}) _≋_
182+
≤-resp= Core.respects₂
183183

184184
≤-trans : IsPartialEquivalence _≈_ _≺_ Respects₂ _≈_ Transitive _≺_
185185
{m n o} Trans (_≤_ {m} {n}) (_≤_ {n} {o}) _≤_
@@ -209,9 +209,9 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
209209
... | inj₁ xs<ys = inj₁ (next x≈y xs<ys)
210210
... | inj₂ xs>ys = inj₂ (next (≈-sym x≈y) xs>ys)
211211

212-
≤-decidable : Decidable _≈_ Decidable _≺_
213-
{m n} Decidable (_≤_ {m} {n})
214-
≤-decidable = Core.decidable (yes tt)
212+
≤-dec : Decidable _≈_ Decidable _≺_
213+
{m n} Decidable (_≤_ {m} {n})
214+
≤-dec = Core.decidable (yes tt)
215215

216216
≤-irrelevant : Irrelevant _≈_ Irrelevant _≺_ Irreflexive _≈_ _≺_
217217
{m n} Irrelevant (_≤_ {m} {n})
@@ -240,7 +240,7 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
240240
≤-isDecPartialOrder ≺-isDecStrictPartialOrder = record
241241
{ isPartialOrder = ≤-isPartialOrder isStrictPartialOrder
242242
; _≟_ = Pointwise.decidable _≟_
243-
; _≤?_ = ≤-decidable _≟_ _<?_
243+
; _≤?_ = ≤-dec _≟_ _<?_
244244
} where open IsDecStrictPartialOrder ≺-isDecStrictPartialOrder
245245

246246
≤-isTotalOrder : IsStrictTotalOrder _≈_ _≺_
@@ -255,7 +255,7 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
255255
≤-isDecTotalOrder ≺-isStrictTotalOrder = record
256256
{ isTotalOrder = ≤-isTotalOrder ≺-isStrictTotalOrder
257257
; _≟_ = Pointwise.decidable _≟_
258-
; _≤?_ = ≤-decidable _≟_ _<?_
258+
; _≤?_ = ≤-dec _≟_ _<?_
259259
} where open IsStrictTotalOrder ≺-isStrictTotalOrder
260260

261261
----------------------------------------------------------------------

0 commit comments

Comments
 (0)