diff -r 06aac7eaec29 -r 71304514891e src/HOL/Combinatorics/Transposition.thy --- a/src/HOL/Combinatorics/Transposition.thy Sun Jun 01 20:01:22 2025 +0200 +++ b/src/HOL/Combinatorics/Transposition.thy Tue Jun 03 12:22:58 2025 +0200 @@ -10,7 +10,7 @@ lemma transpose_apply_first [simp]: \transpose a b a = b\ by (simp add: transpose_def) - + lemma transpose_apply_second [simp]: \transpose a b b = a\ by (simp add: transpose_def) @@ -43,6 +43,9 @@ \transpose a b \ transpose a b = id\ by (rule ext) simp +lemma transpose_eq_id_iff: "Transposition.transpose x y = id \ x = y" + by (auto simp: fun_eq_iff Transposition.transpose_def) + lemma transpose_triple: \transpose a b (transpose b c (transpose a b d)) = transpose a c d\ if \a \ c\ and \b \ c\