summaryrefslogtreecommitdiff
path: root/tests/coq/demo/Demo.v
diff options
context:
space:
mode:
authorSon Ho2024-03-19 05:29:29 +0100
committerSon Ho2024-03-19 05:29:29 +0100
commitf3e16bb43a8ff27a5184d9fa452277cc6a59410f (patch)
treef79760b40b3a9f404b1db0d61f9d452408ef1de5 /tests/coq/demo/Demo.v
parent5a1373f5492f65ff0da6f7e0c34b056a98070908 (diff)
Regenerate the tests
Diffstat (limited to 'tests/coq/demo/Demo.v')
-rw-r--r--tests/coq/demo/Demo.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/tests/coq/demo/Demo.v b/tests/coq/demo/Demo.v
index 48067c02..2fccf6c0 100644
--- a/tests/coq/demo/Demo.v
+++ b/tests/coq/demo/Demo.v
@@ -127,7 +127,7 @@ Definition list_nth_mut1
(T : Type) (n : nat) (l : CList_t T) (i : u32) :
result (T * (T -> result (CList_t T)))
:=
- p <- list_nth_mut1_loop T n l i; let (t, back_'a) := p in Return (t, back_'a)
+ list_nth_mut1_loop T n l i
.
(** [demo::i32_id]: