summaryrefslogtreecommitdiff
path: root/tests/coq/hashmap/Hashmap_FunsExternal_Template.v
blob: ca198a8d666be83a7a3e459c332f050040331a79 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
(** [hashmap]: external functions.
-- This is a template file: rename it to "FunsExternal.lean" and fill the holes. *)
Require Import Primitives.
Import Primitives.
Require Import Coq.ZArith.ZArith.
Require Import List.
Import ListNotations.
Local Open Scope Primitives_scope.
Require Import Hashmap_Types.
Include Hashmap_Types.
Module Hashmap_FunsExternal_Template.

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

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

End Hashmap_FunsExternal_Template.