src/HOL/Library/List_lexord.thy
changeset 22483 86064f2f2188
parent 22316 f662831459de
child 22744 5cbe966d67a2
--- a/src/HOL/Library/List_lexord.thy	Tue Mar 20 15:52:39 2007 +0100
+++ b/src/HOL/Library/List_lexord.thy	Tue Mar 20 15:52:40 2007 +0100
@@ -34,6 +34,12 @@
   apply simp
   done
 
+instance list :: (linorder) distrib_lattice
+  "inf \<equiv> min"
+  "sup \<equiv> max"
+  by intro_classes
+    (auto simp add: inf_list_def sup_list_def min_max.sup_inf_distrib1)
+
 lemma not_less_Nil [simp]: "\<not> (x < [])"
   by (unfold list_less_def) simp