summaryrefslogtreecommitdiff
path: root/tests/coq/hashmap
diff options
context:
space:
mode:
Diffstat (limited to 'tests/coq/hashmap')
-rw-r--r--tests/coq/hashmap/Hashmap_Types.v4
1 files changed, 0 insertions, 4 deletions
diff --git a/tests/coq/hashmap/Hashmap_Types.v b/tests/coq/hashmap/Hashmap_Types.v
index a3b68f9a..ce6e7dab 100644
--- a/tests/coq/hashmap/Hashmap_Types.v
+++ b/tests/coq/hashmap/Hashmap_Types.v
@@ -31,8 +31,4 @@ Arguments Hash_map_max_load_factor {T}.
Arguments Hash_map_max_load {T}.
Arguments Hash_map_slots {T}.
-(** [core::num::u32::{9}::MAX] *)
-Definition core_num_u32_max_body : result u32 := Return (4294967295%u32).
-Definition core_num_u32_max_c : u32 := core_num_u32_max_body%global.
-
End Hashmap_Types .