summaryrefslogtreecommitdiff
path: root/tests/coq/misc/External__Funs.v
diff options
context:
space:
mode:
authorSon Ho2022-11-15 15:25:47 +0100
committerSon HO2022-11-16 15:45:32 +0100
commitfa6dcd3ebbdc7a508157ff2a12f91e70d2012a86 (patch)
treeb72055ef976459079c0f1352a3928bd8a1481f76 /tests/coq/misc/External__Funs.v
parentbd5706896dec0a1aef1accdf51f93af00c5dc6fe (diff)
Change the name of the generated Coq modules
Diffstat (limited to '')
-rw-r--r--tests/coq/misc/External_Funs.v (renamed from tests/coq/misc/External__Funs.v)12
1 files changed, 6 insertions, 6 deletions
diff --git a/tests/coq/misc/External__Funs.v b/tests/coq/misc/External_Funs.v
index e7020040..3ddc1cf3 100644
--- a/tests/coq/misc/External__Funs.v
+++ b/tests/coq/misc/External_Funs.v
@@ -4,11 +4,11 @@ Require Import Primitives.
Import Primitives.
Require Import Coq.ZArith.ZArith.
Local Open Scope Primitives_scope.
-Require Export External__Types.
-Import External__Types.
-Require Export External__Opaque.
-Import External__Opaque.
-Module External__Funs.
+Require Export External_Types.
+Import External_Types.
+Require Export External_Opaque.
+Import External_Opaque.
+Module External_Funs.
(** [external::swap] *)
Definition swap_fwd
@@ -111,4 +111,4 @@ Definition test_swap_non_zero_fwd
if x0 s= 0%u32 then Fail_ Failure else Return (st1, x0)
.
-End External__Funs .
+End External_Funs .