aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/ListSet.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-11 12:41:41 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-11 12:41:41 +0000
commit4ac0580306ea9e45da1863316936d700969465ad (patch)
treebf7595cd76895f3a349e7e75ca9d64231b01dcf8 /theories/Lists/ListSet.v
parent8a7452976731275212f0c464385b380e2d590f5e (diff)
documentation automatique de la bibliothèque standard
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1578 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/ListSet.v')
-rw-r--r--theories/Lists/ListSet.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Lists/ListSet.v b/theories/Lists/ListSet.v
index 565a32404..9af874a3f 100644
--- a/theories/Lists/ListSet.v
+++ b/theories/Lists/ListSet.v
@@ -81,12 +81,12 @@ Section first_definitions.
else (set_add a1 (set_diff x1 y))
end.
- (**
+ (*i
Inductive set_In : A -> set -> Prop :=
set_In_singl : (a:A)(x:set)(set_In a (cons a (nil A)))
| set_In_add : (a,b:A)(x:set)(set_In a x)->(set_In a (set_add b x))
.
- **)
+ i*)
Definition set_In : A -> set -> Prop := (In 1!A).
@@ -324,7 +324,7 @@ Section other_definitions.
Definition set_prod : (set A) -> (set B) -> (set A*B) := (list_prod 1!A 2!B).
- (* B^A, set of applications from A to B *)
+ (* [B^A], set of applications from [A] to [B] *)
Definition set_power : (set A) -> (set B) -> (set (set A*B)) :=
(list_power 1!A 2!B).