src/HOL/List.thy
changeset 15693 3a67e61c6e96
parent 15656 988f91b9c4ef
child 15868 9634b3f9d910
--- a/src/HOL/List.thy	Sun Apr 10 17:20:03 2005 +0200
+++ b/src/HOL/List.thy	Mon Apr 11 12:14:23 2005 +0200
@@ -1909,8 +1909,8 @@
     "lex r == \<Union>n. lexn r n"
         --{*Holds only between lists of the same length*}
 
-  lexico :: "('a \<times> 'a) set => ('a list \<times> 'a list) set"
-    "lexico r == inv_image (less_than <*lex*> lex r) (%xs. (length xs, xs))"
+  lenlex :: "('a \<times> 'a) set => ('a list \<times> 'a list) set"
+    "lenlex r == inv_image (less_than <*lex*> lex r) (%xs. (length xs, xs))"
         --{*Compares lists by their length and then lexicographically*}
 
 
@@ -1952,13 +1952,13 @@
     (\<exists>xys x y xs' ys'. xs = xys @ x # xs' \<and> ys = xys @ y # ys' \<and> (x, y):r)}"
 by (force simp add: lex_def lexn_conv)
 
-lemma wf_lexico [intro!]: "wf r ==> wf (lexico r)"
-by (unfold lexico_def) blast
-
-lemma lexico_conv:
-    "lexico r = {(xs,ys). length xs < length ys |
+lemma wf_lenlex [intro!]: "wf r ==> wf (lenlex r)"
+by (unfold lenlex_def) blast
+
+lemma lenlex_conv:
+    "lenlex r = {(xs,ys). length xs < length ys |
                  length xs = length ys \<and> (xs, ys) : lex r}"
-by (simp add: lexico_def diag_def lex_prod_def measure_def inv_image_def)
+by (simp add: lenlex_def diag_def lex_prod_def measure_def inv_image_def)
 
 lemma Nil_notin_lex [iff]: "([], ys) \<notin> lex r"
 by (simp add: lex_conv)