| author | wenzelm | 
| Thu, 11 Nov 1999 11:29:11 +0100 | |
| changeset 8008 | 8916ea9ec178 | 
| parent 6810 | 731c848f6f0c | 
| child 12338 | de0f4a63baa5 | 
| permissions | -rw-r--r-- | 
(* 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 = GenPrefix + instance list :: (term) order (prefix_refl,prefix_trans,prefix_antisym,prefix_less_le) end