aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/import_mod.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-12-21 23:50:17 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-12-21 23:50:17 +0000
commit4d4f08acb5e5f56d38289e5629173bc1b8b5fd57 (patch)
treec160d442d54dbd15cbd0ab3500cdf94d0a6da74e /test-suite/success/import_mod.v
parent960859c0c10e029f9768d0d70addeca8f6b6d784 (diff)
Abandon tests syntaxe v7; remplacement des .v par des fichiers en syntaxe v8
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@7693 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/import_mod.v')
-rw-r--r--test-suite/success/import_mod.v36
1 files changed, 18 insertions, 18 deletions
diff --git a/test-suite/success/import_mod.v b/test-suite/success/import_mod.v
index b4a8af46f..c098c6e89 100644
--- a/test-suite/success/import_mod.v
+++ b/test-suite/success/import_mod.v
@@ -1,38 +1,38 @@
-Definition p:=O.
-Definition m:=O.
+Definition p := 0.
+Definition m := 0.
Module Test_Import.
Module P.
- Definition p:=(S O).
+ Definition p := 1.
End P.
Module M.
Import P.
- Definition m:=p.
+ Definition m := p.
End M.
Module N.
Import M.
- Lemma th0 : p=O.
- Reflexivity.
+ Lemma th0 : p = 0.
+ reflexivity.
Qed.
End N.
(* M and P should be closed *)
- Lemma th1 : m=O /\ p=O.
- Split; Reflexivity.
+ Lemma th1 : m = 0 /\ p = 0.
+ split; reflexivity.
Qed.
Import N.
(* M and P should still be closed *)
- Lemma th2 : m=O /\ p=O.
- Split; Reflexivity.
+ Lemma th2 : m = 0 /\ p = 0.
+ split; reflexivity.
Qed.
End Test_Import.
@@ -42,34 +42,34 @@ End Test_Import.
Module Test_Export.
Module P.
- Definition p:=(S O).
+ Definition p := 1.
End P.
Module M.
Export P.
- Definition m:=p.
+ Definition m := p.
End M.
Module N.
Export M.
- Lemma th0 : p=(S O).
- Reflexivity.
+ Lemma th0 : p = 1.
+ reflexivity.
Qed.
End N.
(* M and P should be closed *)
- Lemma th1 : m=O /\ p=O.
- Split; Reflexivity.
+ Lemma th1 : m = 0 /\ p = 0.
+ split; reflexivity.
Qed.
Import N.
(* M and P should now be opened *)
- Lemma th2 : m=(S O) /\ p=(S O).
- Split; Reflexivity.
+ Lemma th2 : m = 1 /\ p = 1.
+ split; reflexivity.
Qed.
End Test_Export.