changeset 30971 | 7fbebf75b3ef |
parent 30952 | 7ab2716dd93b |
child 31022 | a438b4516dd3 |
--- a/src/HOL/List.thy Fri Apr 24 08:24:54 2009 +0200 +++ b/src/HOL/List.thy Fri Apr 24 17:45:15 2009 +0200 @@ -198,7 +198,7 @@ definition rotate :: "nat \<Rightarrow> 'a list \<Rightarrow> 'a list" where - "rotate n = rotate1 o^ n" + "rotate n = rotate1 ^^ n" definition list_all2 :: "('a => 'b => bool) => 'a list => 'b list => bool" where