src/HOL/UNITY/ListOrder.thy
changeset 6810 731c848f6f0c
parent 6708 62beb3336b02
child 12338 de0f4a63baa5
--- a/src/HOL/UNITY/ListOrder.thy	Thu Jun 10 10:38:11 1999 +0200
+++ b/src/HOL/UNITY/ListOrder.thy	Thu Jun 10 10:38:41 1999 +0200
@@ -6,7 +6,7 @@
 Lists are partially ordered by the prefix relation
 *)
 
-ListOrder = Prefix +
+ListOrder = GenPrefix +
 
 instance list :: (term) order
     (prefix_refl,prefix_trans,prefix_antisym,prefix_less_le)