aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/ListSet.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-15 12:43:02 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-15 12:43:02 +0000
commitf064defc1387c251540361b19f0af751d21c0f82 (patch)
treec8b5db50ab4e176c9c8224079ca23f8157b0b6c7 /theories/Lists/ListSet.v
parent60568746faf8286afd3554d46a0f0db0345c2704 (diff)
Nettoyage argument de nil
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4639 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/ListSet.v')
-rw-r--r--theories/Lists/ListSet.v10
1 files changed, 6 insertions, 4 deletions
diff --git a/theories/Lists/ListSet.v b/theories/Lists/ListSet.v
index 77f943716..4b7083c0a 100644
--- a/theories/Lists/ListSet.v
+++ b/theories/Lists/ListSet.v
@@ -19,6 +19,7 @@
Require PolyList.
Set Implicit Arguments.
+V7only [Implicits nil [1].].
Section first_definitions.
@@ -27,11 +28,11 @@ Section first_definitions.
Definition set := (list A).
- Definition empty_set := (nil ?) : set.
+ Definition empty_set := (!nil ?) : set.
Fixpoint set_add [a:A; x:set] : set :=
Cases x of
- | nil => (cons a (nil A))
+ | nil => (cons a nil)
| (cons a1 x1) => Cases (Aeq_dec a a1) of
| (left _) => (cons a1 x1)
| (right _) => (cons a1 (set_add a x1))
@@ -60,7 +61,7 @@ Section first_definitions.
Fixpoint set_inter [x:set] : set -> set :=
Cases x of
- | nil => [y](nil A)
+ | nil => [y]nil
| (cons a1 x1) => [y]if (set_mem a1 y)
then (cons a1 (set_inter x1 y))
else (set_inter x1 y)
@@ -75,7 +76,7 @@ Section first_definitions.
(** returns the set of all els of [x] that does not belong to [y] *)
Fixpoint set_diff [x:set] : set -> set :=
[y]Cases x of
- | nil => (nil A)
+ | nil => nil
| (cons a1 x1) => if (set_mem a1 y)
then (set_diff x1 y)
else (set_add a1 (set_diff x1 y))
@@ -384,4 +385,5 @@ Section other_definitions.
End other_definitions.
+V7only [Implicits nil [].].
Unset Implicit Arguments.