equal
deleted
inserted
replaced
889 by (auto simp: bij_betw_def) |
889 by (auto simp: bij_betw_def) |
890 |
890 |
891 lemma bij_swap_iff [simp]: "bij (swap a b f) \<longleftrightarrow> bij f" |
891 lemma bij_swap_iff [simp]: "bij (swap a b f) \<longleftrightarrow> bij f" |
892 by simp |
892 by simp |
893 |
893 |
|
894 subsection \<open>Transpositions\<close> |
|
895 |
|
896 lemma swap_id_idempotent [simp]: "Fun.swap a b id \<circ> Fun.swap a b id = id" |
|
897 by (rule ext) (auto simp add: Fun.swap_def) |
|
898 |
|
899 lemma swap_id_eq: "Fun.swap a b id x = (if x = a then b else if x = b then a else x)" |
|
900 by (simp add: Fun.swap_def) |
|
901 |
|
902 lemma bij_swap_compose_bij: |
|
903 \<open>bij (Fun.swap a b id \<circ> p)\<close> if \<open>bij p\<close> |
|
904 using that by (rule bij_comp) simp |
|
905 |
894 hide_const (open) swap |
906 hide_const (open) swap |
895 |
907 |
896 |
908 |
897 subsection \<open>Inversion of injective functions\<close> |
909 subsection \<open>Inversion of injective functions\<close> |
898 |
910 |