src/HOL/UNITY/Rename.thy
changeset 47448 e5438c5797ae
parent 46476 a89b4bc311a5
child 59180 85ec71012df8
equal deleted inserted replaced
47447:ae9286f64574 47448:e5438c5797ae
    62 apply (rule Extend.inj_extend_act)
    62 apply (rule Extend.inj_extend_act)
    63 apply simp
    63 apply simp
    64 apply (simp add: bij_extend_act_eq_project_act)
    64 apply (simp add: bij_extend_act_eq_project_act)
    65 apply (rule surjI)
    65 apply (rule surjI)
    66 apply (rule Extend.extend_act_inverse)
    66 apply (rule Extend.extend_act_inverse)
    67 apply (blast intro: bij_imp_bij_inv good_map_bij)
    67 apply (blast intro: bij_imp_bij_inv)
    68 done
    68 done
    69 
    69 
    70 lemma bij_project_act: "bij h ==> bij (project_act (%(x,u::'c). h x))"
    70 lemma bij_project_act: "bij h ==> bij (project_act (%(x,u::'c). h x))"
    71 apply (frule bij_imp_bij_inv [THEN bij_extend_act])
    71 apply (frule bij_imp_bij_inv [THEN bij_extend_act])
    72 apply (simp add: bij_extend_act_eq_project_act bij_imp_bij_inv inv_inv_eq)
    72 apply (simp add: bij_extend_act_eq_project_act bij_imp_bij_inv inv_inv_eq)