diff options
| author | Hugo Herbelin | 2020-08-18 22:49:00 +0200 |
|---|---|---|
| committer | Hugo Herbelin | 2020-10-05 16:19:12 +0200 |
| commit | 2fb42ce6b9b74a2c5f66e9fa9cb16745cdb85687 (patch) | |
| tree | 88d12d5f428c1dc89cb8cb272e3531a2d7a531de /theories/Strings/ByteVector.v | |
| parent | 571834b2b43e4281ef4940ee5894d8191588bb6c (diff) | |
Adapting theories to unused pattern-matching variable warning.
Diffstat (limited to 'theories/Strings/ByteVector.v')
| -rw-r--r-- | theories/Strings/ByteVector.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Strings/ByteVector.v b/theories/Strings/ByteVector.v index ac0323442a..144ffd59e0 100644 --- a/theories/Strings/ByteVector.v +++ b/theories/Strings/ByteVector.v @@ -42,7 +42,7 @@ Fixpoint to_Bvector {n : nat} (v : ByteVector n) : Bvector (n * 8) := Fixpoint of_Bvector {n : nat} : Bvector (n * 8) -> ByteVector n := match n with | 0 => fun _ => [] - | S n' => + | S _ => fun v => let (b0, v1) := uncons v in let (b1, v2) := uncons v1 in |
