summaryrefslogtreecommitdiff
path: root/tests/coq/arrays
diff options
context:
space:
mode:
authorSon Ho2024-04-25 16:28:30 +0200
committerSon Ho2024-04-25 16:28:30 +0200
commit036756d6bddbcf9bc936489779ed36c7e4d22d14 (patch)
tree01ab1e2e5d1bbbbceedb6683d0826f05bd0a5720 /tests/coq/arrays
parenteb5b2e76de6e2c6780b9817c1424777276ea5e00 (diff)
Regenerate and fix the tests
Diffstat (limited to 'tests/coq/arrays')
-rw-r--r--tests/coq/arrays/Primitives.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/tests/coq/arrays/Primitives.v b/tests/coq/arrays/Primitives.v
index 5ffda12f..b29fce43 100644
--- a/tests/coq/arrays/Primitives.v
+++ b/tests/coq/arrays/Primitives.v
@@ -564,6 +564,13 @@ Definition core_clone_CloneI128 : core_clone_Clone i128 := {|
clone := fun x => Ok (core_clone_impls_CloneI128_clone x)
|}.
+(** [core::option::{core::option::Option<T>}::unwrap] *)
+Definition core_option_Option_unwrap (T : Type) (x : option T) : result T :=
+ match x with
+ | None => Fail_ Failure
+ | Some x => Ok x
+ end.
+
(*** core::ops *)
(* Trait declaration: [core::ops::index::Index] *)