aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Wellfounded/Lexicographic_Exponentiation.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Wellfounded/Lexicographic_Exponentiation.v')
-rw-r--r--theories/Wellfounded/Lexicographic_Exponentiation.v8
1 files changed, 5 insertions, 3 deletions
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.