aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/ListSet.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-09 22:07:35 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-09 22:07:35 +0000
commitccd3cc391a15be9b59a3fc3646a3dae1328fbc64 (patch)
tree2bbd0f4c2f8a89095724814b0917eeae36742779 /theories/Lists/ListSet.v
parent9c695ca0d906454c127285fe465f219eef01bed3 (diff)
cast de nil
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3897 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/ListSet.v')
-rw-r--r--theories/Lists/ListSet.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Lists/ListSet.v b/theories/Lists/ListSet.v
index a72adbb21..77f943716 100644
--- a/theories/Lists/ListSet.v
+++ b/theories/Lists/ListSet.v
@@ -27,7 +27,7 @@ Section first_definitions.
Definition set := (list A).
- Definition empty_set := (nil A).
+ Definition empty_set := (nil ?) : set.
Fixpoint set_add [a:A; x:set] : set :=
Cases x of