Skip to content

Commit 8c5066b

Browse files
authored
fixed issue #602 for vectors, too (#1672)
1 parent b3bb7b4 commit 8c5066b

File tree

2 files changed

+9
-1
lines changed

2 files changed

+9
-1
lines changed

CHANGELOG.md

+5
Original file line numberDiff line numberDiff line change
@@ -1014,6 +1014,11 @@ Other minor changes
10141014
transpose-replicate : transpose (replicate xs) ≡ map replicate xs
10151015
```
10161016

1017+
* Added new proofs in `Data.Vec.Relation.Binary.Lex.Strict`:
1018+
```agda
1019+
xs≮[] : ∀ {n} (xs : Vec A n) → ¬ xs < []
1020+
```
1021+
10171022
* Added new functions in `Data.Vec.Relation.Unary.All`:
10181023
```
10191024
decide : Π[ P ∪ Q ] → Π[ All P ∪ Any Q ]

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

+4-1
Original file line numberDiff line numberDiff line change
@@ -60,8 +60,11 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
6060
_≋_ = Pointwise _≈_
6161
_<_ = Lex-< _≈_ _≺_
6262

63+
xs≮[] : {n} (xs : Vec A n) ¬ xs < []
64+
xs≮[] _ (base ())
65+
6366
¬[]<[] : ¬ [] < []
64-
¬[]<[] (base ())
67+
¬[]<[] = xs≮[] []
6568

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

0 commit comments

Comments
 (0)