aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/Array.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/hls/Array.v')
-rw-r--r--src/hls/Array.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/src/hls/Array.v b/src/hls/Array.v
index 0f5ae02..de74611 100644
--- a/src/hls/Array.v
+++ b/src/hls/Array.v
@@ -190,7 +190,10 @@ Proof.
auto using nth_error_nth.
Qed.
-(** Tail recursive version of standard library function. *)
+(*|
+Tail recursive version of standard library function.
+|*)
+
Fixpoint list_repeat' {A : Type} (acc : list A) (a : A) (n : nat) : list A :=
match n with
| O => acc