aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/import_lib.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success/import_lib.v')
-rw-r--r--test-suite/success/import_lib.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/test-suite/success/import_lib.v b/test-suite/success/import_lib.v
index b35436247..d031691d8 100644
--- a/test-suite/success/import_lib.v
+++ b/test-suite/success/import_lib.v
@@ -115,7 +115,7 @@ Module Test_Import.
Qed.
End Test_Import.
-(***********************************************************************)
+(************************************************************************)
Module Test_Export.
Module M.
@@ -156,7 +156,7 @@ Module Test_Export.
End Test_Export.
-(***********************************************************************)
+(************************************************************************)
Module Test_Require_Export.