src/ZF/Perm.thy
changeset 13185 da61bfa0a391
parent 13180 a82610e49b2d
child 13269 3ba9be497c33
equal deleted inserted replaced
13184:197e5a88c9df 13185:da61bfa0a391
   566 val id_inj = thm "id_inj";
   566 val id_inj = thm "id_inj";
   567 val id_surj = thm "id_surj";
   567 val id_surj = thm "id_surj";
   568 val id_bij = thm "id_bij";
   568 val id_bij = thm "id_bij";
   569 val subset_iff_id = thm "subset_iff_id";
   569 val subset_iff_id = thm "subset_iff_id";
   570 val inj_converse_fun = thm "inj_converse_fun";
   570 val inj_converse_fun = thm "inj_converse_fun";
   571 val left_inverse_lemma = thm "left_inverse_lemma";
       
   572 val left_inverse = thm "left_inverse";
   571 val left_inverse = thm "left_inverse";
   573 val left_inverse_bij = thm "left_inverse_bij";
   572 val left_inverse_bij = thm "left_inverse_bij";
   574 val right_inverse_lemma = thm "right_inverse_lemma";
       
   575 val right_inverse = thm "right_inverse";
   573 val right_inverse = thm "right_inverse";
   576 val right_inverse_bij = thm "right_inverse_bij";
   574 val right_inverse_bij = thm "right_inverse_bij";
   577 val inj_converse_inj = thm "inj_converse_inj";
   575 val inj_converse_inj = thm "inj_converse_inj";
   578 val inj_converse_surj = thm "inj_converse_surj";
   576 val inj_converse_surj = thm "inj_converse_surj";
   579 val bij_converse_bij = thm "bij_converse_bij";
   577 val bij_converse_bij = thm "bij_converse_bij";