aboutsummaryrefslogtreecommitdiff
path: root/src/Galois/BaseSystem.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Galois/BaseSystem.v')
-rw-r--r--src/Galois/BaseSystem.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Galois/BaseSystem.v b/src/Galois/BaseSystem.v
index 8197bed8d..28ae37233 100644
--- a/src/Galois/BaseSystem.v
+++ b/src/Galois/BaseSystem.v
@@ -39,7 +39,7 @@ Module BaseSystem (Import B:BaseCoefs).
Lemma decode'_truncate : forall bs us, decode' bs us = decode' bs (firstn (length bs) us).
Proof.
- unfold decode, decode'; intros; f_equal; apply combine_truncate_l.
+ unfold decode'; intros; f_equal; apply combine_truncate_l.
Qed.
Fixpoint add (us vs:digits) : digits :=