Nominal/Nominal2_FSet.thy
changeset 2542 1f5c8e85c41f
parent 2540 135ac0fb2686
child 2550 551c5a8b6b2c
equal deleted inserted replaced
2541:d7269488c4b5 2542:1f5c8e85c41f
    70   apply (rule fset_finite_supp)
    70   apply (rule fset_finite_supp)
    71   done
    71   done
    72 
    72 
    73 lemma atom_map_fset_cong:
    73 lemma atom_map_fset_cong:
    74   shows "map_fset atom x = map_fset atom y \<longleftrightarrow> x = y"
    74   shows "map_fset atom x = map_fset atom y \<longleftrightarrow> x = y"
    75   apply(rule inj_map_fset_eq_iff)
    75   apply(rule inj_map_fset_cong)
    76   apply(simp add: inj_on_def)
    76   apply(simp add: inj_on_def)
    77   done
    77   done
    78 
    78 
    79 lemma supp_map_fset_atom:
    79 lemma supp_map_fset_atom:
    80   shows "supp (map_fset atom S) = supp S"
    80   shows "supp (map_fset atom S) = supp S"