diff -r 6061ae1f90f2 -r 9bc16273c2d4 src/HOL/UNITY/ListOrder.thy --- a/src/HOL/UNITY/ListOrder.thy Fri Jun 17 11:35:35 2005 +0200 +++ b/src/HOL/UNITY/ListOrder.thy Fri Jun 17 16:12:49 2005 +0200 @@ -15,7 +15,7 @@ header {*The Prefix Ordering on Lists*} -theory ListOrder = Main: +theory ListOrder imports Main begin consts genPrefix :: "('a * 'a)set => ('a list * 'a list)set"