src/HOL/UNITY/ListOrder.thy
changeset 6708 62beb3336b02
child 6810 731c848f6f0c
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/UNITY/ListOrder.thy	Mon May 24 15:47:57 1999 +0200
@@ -0,0 +1,14 @@
+(*  Title:      HOL/UNITY/ListOrder
+    ID:         $Id$
+    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
+    Copyright   1998  University of Cambridge
+
+Lists are partially ordered by the prefix relation
+*)
+
+ListOrder = Prefix +
+
+instance list :: (term) order
+    (prefix_refl,prefix_trans,prefix_antisym,prefix_less_le)
+
+end