mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-11 14:48:42 +00:00
Lots of refactoring towards partially-ordered ring R (#109)
This commit is contained in:
@@ -13,6 +13,9 @@ record Sequence {a : _} (A : Set a) : Set a where
|
||||
head : A
|
||||
tail : Sequence A
|
||||
|
||||
headInjective : {a : _} {A : Set a} {s1 s2 : Sequence A} → s1 ≡ s2 → Sequence.head s1 ≡ Sequence.head s2
|
||||
headInjective {s1 = s1} {.s1} refl = refl
|
||||
|
||||
constSequence : {a : _} {A : Set a} (k : A) → Sequence A
|
||||
Sequence.head (constSequence k) = k
|
||||
Sequence.tail (constSequence k) = constSequence k
|
||||
|
Reference in New Issue
Block a user