File tree 2 files changed +9
-1
lines changed
src/Data/Vec/Relation/Binary/Lex
2 files changed +9
-1
lines changed Original file line number Diff line number Diff line change @@ -1014,6 +1014,11 @@ Other minor changes
1014
1014
transpose-replicate : transpose (replicate xs) ≡ map replicate xs
1015
1015
```
1016
1016
1017
+ * Added new proofs in ` Data.Vec.Relation.Binary.Lex.Strict ` :
1018
+ ``` agda
1019
+ xs≮[] : ∀ {n} (xs : Vec A n) → ¬ xs < []
1020
+ ```
1021
+
1017
1022
* Added new functions in ` Data.Vec.Relation.Unary.All ` :
1018
1023
```
1019
1024
decide : Π[ P ∪ Q ] → Π[ All P ∪ Any Q ]
Original file line number Diff line number Diff line change @@ -60,8 +60,11 @@ module _ {_≈_ : Rel A ℓ₁} {_≺_ : Rel A ℓ₂} where
60
60
_≋_ = Pointwise _≈_
61
61
_<_ = Lex-< _≈_ _≺_
62
62
63
+ xs≮[] : ∀ {n} (xs : Vec A n) → ¬ xs < []
64
+ xs≮[] _ (base ())
65
+
63
66
¬[]<[] : ¬ [] < []
64
- ¬[]<[] (base ())
67
+ ¬[]<[] = xs≮[] []
65
68
66
69
module _ (≺-irrefl : Irreflexive _≈_ _≺_) where
67
70
You can’t perform that action at this time.
0 commit comments