From 97621f6e9c6a23a839bf0a2f28efec9434a158a8 Mon Sep 17 00:00:00 2001 From: herbelin Date: Fri, 19 Sep 2003 00:07:57 +0000 Subject: Ajout notation :: pour cons git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4418 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Lists/PolyList.v | 9 +++++++-- 1 file changed, 7 insertions(+), 2 deletions(-) (limited to 'theories/Lists/PolyList.v') 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. -- cgit v1.2.3