Skip to content
Merged
Show file tree
Hide file tree
Changes from 1 commit
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
2 changes: 1 addition & 1 deletion CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -2686,7 +2686,7 @@ Other minor changes

* Added new proofs in `Data.Vec.Relation.Binary.Lex.Strict`:
```agda
xs≮[] : ∀ {n} (xs : Vec A n) → ¬ xs < []
xs≮[] : ∀ {n} {xs : Vec A n} → ¬ xs < []
<-respectsˡ : IsPartialEquivalence _≈_ → _≺_ Respectsˡ _≈_ →
∀ {m n} → _Respectsˡ_ (_<_ {m} {n}) _≋_
<-respectsʳ : IsPartialEquivalence _≈_ → _≺_ Respectsʳ _≈_ →
Expand Down
6 changes: 3 additions & 3 deletions src/Data/List/Relation/Binary/Lex/Strict.agda
Original file line number Diff line number Diff line change
Expand Up @@ -45,11 +45,11 @@ module _ {a ℓ₁ ℓ₂} {A : Set a} where
_≋_ = Pointwise _≈_
_<_ = Lex-< _≈_ _≺_

xs≮[] : ∀ xs → ¬ xs < []
xs≮[] _ (base ())
xs≮[] : ∀ {xs} → ¬ xs < []
xs≮[] (base ())

¬[]<[] : ¬ [] < []
¬[]<[] = xs≮[] []
¬[]<[] = xs≮[]

<-irreflexive : Irreflexive _≈_ _≺_ → Irreflexive _≋_ _<_
<-irreflexive irr (x≈y ∷ xs≋ys) (this x<y) = irr x≈y x<y
Expand Down
8 changes: 4 additions & 4 deletions src/Data/Vec/Relation/Binary/Lex/Strict.agda
Original file line number Diff line number Diff line change
Expand Up @@ -63,11 +63,11 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
_≋_ = Pointwise _≈_
_<_ = Lex-< _≈_ _≺_

xs≮[] : ∀ {n} (xs : Vec A n) → ¬ xs < []
xs≮[] _ (base ())
xs≮[] : ∀ {n} {xs : Vec A n} → ¬ xs < []
xs≮[] (base ())

¬[]<[] : ¬ [] < []
¬[]<[] = xs≮[] []
¬[]<[] = xs≮[]

module _ (≺-irrefl : Irreflexive _≈_ _≺_) where

Expand Down Expand Up @@ -128,7 +128,7 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
where

<-wellFounded : ∀ {n} → WellFounded (_<_ {n})
<-wellFounded {0} [] = acc λ ys ys<[] → ⊥-elim (xs≮[] ys ys<[])
<-wellFounded {0} [] = acc λ ys ys<[] → ⊥-elim (xs≮[] ys<[])
<-wellFounded {suc n} xs = Subrelation.wellFounded <⇒uncons-Lex uncons-Lex-wellFounded xs
where
<⇒uncons-Lex : {xs ys : Vec A (suc n)} → xs < ys → (×-Lex _≈_ _≺_ _<_ on uncons) xs ys
Expand Down