summaryrefslogtreecommitdiff
path: root/tests/coq/hashmap_main/HashmapMain_FunsExternal_Template.v
diff options
context:
space:
mode:
authorGuillaume Boisseau2024-05-28 11:56:39 +0200
committerGitHub2024-05-28 11:56:39 +0200
commitef7792c106a1f33397c206fcb5124b5ddfe64378 (patch)
treea72fae46702fc4c2eb32e1361a2538eb7a5f5545 /tests/coq/hashmap_main/HashmapMain_FunsExternal_Template.v
parent4f26c7f6f1e554d8ec2f46e868d5dc66c4160d16 (diff)
parentc4d2af051c18c4c81b1e57a45210c37c89c8330f (diff)
Merge pull request #213 from AeneasVerif/cleanup-tests
Diffstat (limited to 'tests/coq/hashmap_main/HashmapMain_FunsExternal_Template.v')
-rw-r--r--tests/coq/hashmap_main/HashmapMain_FunsExternal_Template.v26
1 files changed, 0 insertions, 26 deletions
diff --git a/tests/coq/hashmap_main/HashmapMain_FunsExternal_Template.v b/tests/coq/hashmap_main/HashmapMain_FunsExternal_Template.v
deleted file mode 100644
index 66835e8c..00000000
--- a/tests/coq/hashmap_main/HashmapMain_FunsExternal_Template.v
+++ /dev/null
@@ -1,26 +0,0 @@
-(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
-(** [hashmap_main]: 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 HashmapMain_Types.
-Include HashmapMain_Types.
-Module HashmapMain_FunsExternal_Template.
-
-(** [hashmap_main::hashmap_utils::deserialize]:
- Source: 'tests/src/hashmap_utils.rs', lines 11:0-11:43 *)
-Axiom hashmap_utils_deserialize
- : state -> result (state * (hashmap_HashMap_t u64))
-.
-
-(** [hashmap_main::hashmap_utils::serialize]:
- Source: 'tests/src/hashmap_utils.rs', lines 6:0-6:42 *)
-Axiom hashmap_utils_serialize
- : hashmap_HashMap_t u64 -> state -> result (state * unit)
-.
-
-End HashmapMain_FunsExternal_Template.