diff -r 8dbc521ee97f -r 28bb34eeedc5 QuotList.thy --- a/QuotList.thy Fri Dec 04 09:10:31 2009 +0100 +++ b/QuotList.thy Fri Dec 04 09:18:46 2009 +0100 @@ -15,7 +15,7 @@ | "LIST_REL R (x#xs) (y#ys) = (R x y \ LIST_REL R xs ys)" lemma LIST_REL_EQ: - shows "LIST_REL (op =) = (op =)" + shows "LIST_REL (op =) \ (op =)" unfolding expand_fun_eq apply(rule allI)+ apply(induct_tac x xa rule: list_induct2')