summaryrefslogtreecommitdiff
path: root/tests/coq/hashmap/Hashmap_FunsExternal.v
blob: bcf12c17ec3039ddd62b5f4fed732066957a58f3 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
(** [hashmap]: external functions. *)
Require Import Primitives.
Import Primitives.
Require Import Coq.ZArith.ZArith.
Require Import List.
Import ListNotations.
Local Open Scope Primitives_scope.
Require Export Hashmap_Types.
Import Hashmap_Types.
Module Hashmap_FunsExternal.

(** [hashmap::hashmap_utils::deserialize]:
    Source: 'tests/src/hashmap.rs', lines 330:4-330:47 *)
Axiom hashmap_utils_deserialize : state -> result (state * (HashMap_t u64)).

(** [hashmap::hashmap_utils::serialize]:
    Source: 'tests/src/hashmap.rs', lines 325:4-325:46 *)
Axiom hashmap_utils_serialize : HashMap_t u64 -> state -> result (state * unit)
.

End Hashmap_FunsExternal.