From cb1ae314411d78952062e5092804b85d981ad6e1 Mon Sep 17 00:00:00 2001 From: barras Date: Wed, 12 Mar 2003 17:49:21 +0000 Subject: *** empty log message *** git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3761 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Wellfounded/Lexicographic_Exponentiation.v | 8 +++++--- 1 file changed, 5 insertions(+), 3 deletions(-) (limited to 'theories/Wellfounded') diff --git a/theories/Wellfounded/Lexicographic_Exponentiation.v b/theories/Wellfounded/Lexicographic_Exponentiation.v index 5c73cdae0..8efa124c3 100644 --- a/theories/Wellfounded/Lexicographic_Exponentiation.v +++ b/theories/Wellfounded/Lexicographic_Exponentiation.v @@ -32,7 +32,10 @@ Notation List := (list A). Notation Nil := (nil A). (* useless but symmetric *) Notation Cons := (cons 1!A). +Notation "<< x , y >>" := (exist List Descl x y) (at level 0) + V8only (at level 0, x,y at level 100). +V7only[ Syntax constr level 1: List [ (list A) ] -> ["List"] @@ -42,12 +45,11 @@ Syntax constr level 10: Cons2 [ (cons A $e $l) ] -> ["Cons " $e:L " " $l:L ]. -Hints Resolve d_one d_nil t_step. - Syntax constr level 1: pair_sig [ (exist (list A) Desc $e $d) ] -> ["<<" $e:L "," $d:L ">>"]. - +]. +Hints Resolve d_one d_nil t_step. Lemma left_prefix : (x,y,z:List)(ltl x^y z)-> (ltl x z). Proof. -- cgit v1.2.3