diff -r 23a8c5ac35f8 -r 69916a850301 src/ZF/UNITY/GenPrefix.thy --- a/src/ZF/UNITY/GenPrefix.thy Sat Oct 17 01:05:59 2009 +0200 +++ b/src/ZF/UNITY/GenPrefix.thy Sat Oct 17 14:43:18 2009 +0200 @@ -1,10 +1,10 @@ -(* ID: $Id$ +(* Title: ZF/UNITY/GenPrefix.thy Author: Sidi O Ehmety, Cambridge University Computer Laboratory Copyright 2001 University of Cambridge - :gen_prefix(r) - if ys = xs' @ zs where length(xs) = length(xs') - and corresponding elements of xs, xs' are pairwise related by r +:gen_prefix(r) + if ys = xs' @ zs where length(xs) = length(xs') + and corresponding elements of xs, xs' are pairwise related by r Based on Lex/Prefix *) @@ -31,10 +31,10 @@ Nil: "<[],[]>:gen_prefix(A, r)" prepend: "[| :gen_prefix(A, r); :r; x:A; y:A |] - ==> : gen_prefix(A, r)" + ==> : gen_prefix(A, r)" append: "[| :gen_prefix(A, r); zs:list(A) |] - ==> :gen_prefix(A, r)" + ==> :gen_prefix(A, r)" type_intros app_type list.Nil list.Cons definition