diff -r e44d86131648 -r 0c18df79b1c8 src/ZF/ex/Commutation.thy --- a/src/ZF/ex/Commutation.thy Tue Sep 27 16:51:35 2022 +0100 +++ b/src/ZF/ex/Commutation.thy Tue Sep 27 17:03:23 2022 +0100 @@ -1,5 +1,5 @@ (* Title: ZF/ex/Commutation.thy - Author: Tobias Nipkow & Sidi Ould Ehmety + Author: Tobias Nipkow \ Sidi Ould Ehmety Copyright 1995 TU Muenchen Commutation theory for proving the Church Rosser theorem. @@ -10,7 +10,7 @@ definition square :: "[i, i, i, i] => o" where "square(r,s,t,u) \ - (\a b. \ r \ (\c. \ s \ (\x. \ t & \ u)))" + (\a b. \ r \ (\c. \ s \ (\x. \ t \ \ u)))" definition commute :: "[i, i] => o" where @@ -27,7 +27,7 @@ definition Church_Rosser :: "i => o" where "Church_Rosser(r) \ (\x y. \ (r \ converse(r))^* \ - (\z. \ r^* & \ r^*))" + (\z. \ r^* \ \ r^*))" definition confluent :: "i=>o" where