aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/modules/Tescik.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/modules/Tescik.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/modules/Tescik.v')
-rw-r--r--test-suite/modules/Tescik.v32
1 files changed, 16 insertions, 16 deletions
diff --git a/test-suite/modules/Tescik.v b/test-suite/modules/Tescik.v
index 13c284181..8dadace77 100644
--- a/test-suite/modules/Tescik.v
+++ b/test-suite/modules/Tescik.v
@@ -1,30 +1,30 @@
Module Type ELEM.
- Parameter A:Set.
- Parameter x:A.
+ Parameter A : Set.
+ Parameter x : A.
End ELEM.
Module Nat.
- Definition A:=nat.
- Definition x:=O.
+ Definition A := nat.
+ Definition x := 0.
End Nat.
-Module List[X:ELEM].
- Inductive list : Set := nil : list
- | cons : X.A -> list -> list.
+Module List (X: ELEM).
+ Inductive list : Set :=
+ | nil : list
+ | cons : X.A -> list -> list.
- Definition head :=
- [l:list]Cases l of
- nil => X.x
- | (cons x _) => x
- end.
+ Definition head (l : list) := match l with
+ | nil => X.x
+ | cons x _ => x
+ end.
- Definition singl := [x:X.A] (cons x nil).
+ Definition singl (x : X.A) := cons x nil.
- Lemma head_singl : (x:X.A)(head (singl x))=x.
- Auto.
+ Lemma head_singl : forall x : X.A, head (singl x) = x.
+ auto.
Qed.
End List.
-Module N:=(List Nat).
+Module N := List Nat. \ No newline at end of file