aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/import_lib.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-07-16 20:01:26 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-07-16 20:01:26 +0000
commit763cf4f37e10d9a0e8a2a0e9286c02708a60bf08 (patch)
tree006f610487a8a2557176d085852d3e443c547493 /test-suite/success/import_lib.v
parent3e430c449809e6db5c20c2b5b57fafdd5a230fd3 (diff)
Nouvelle en-tĂȘte
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5920 85f007b7-540e-0410-9357-904b9bb8a0f7
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.