aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/PolyList.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-19 00:07:57 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-19 00:07:57 +0000
commit97621f6e9c6a23a839bf0a2f28efec9434a158a8 (patch)
treebcedab9dfd779dc19a8d1ec28c86c8a99ede82dd /theories/Lists/PolyList.v
parent55ef6bcc3bb3995f542b56efacae4f69693d71d4 (diff)
Ajout notation :: pour cons
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4418 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/PolyList.v')
-rw-r--r--theories/Lists/PolyList.v9
1 files changed, 7 insertions, 2 deletions
diff --git a/theories/Lists/PolyList.v b/theories/Lists/PolyList.v
index cdc0f3655..57ed3ec2d 100644
--- a/theories/Lists/PolyList.v
+++ b/theories/Lists/PolyList.v
@@ -22,6 +22,11 @@ Inductive list : Set := nil : list | cons : A -> list -> list.
Unset Contextual Implicits.
+Infix "::" cons (at level 7, right associativity) : list_scope
+ V8only (at level 45, right associativity).
+
+Open Scope list_scope.
+
(*************************)
(** Discrimination *)
(*************************)
@@ -41,8 +46,8 @@ Fixpoint app [l:list] : list -> list
| (cons a l1) => (cons a (app l1 m))
end.
-Infix RIGHTA 7 "^" app
- V8only 30.
+Infix RIGHTA 7 "^" app : list_scope
+ V8only 45.
Lemma app_nil_end : (l:list)l=(l^nil).
Proof.