src/HOL/Library/Quotient_Set.thy
changeset 44873 045fedcfadf6
parent 44459 079ccfb074d9
child 45970 b6d0cff57d96
equal deleted inserted replaced
44870:0d23a8ae14df 44873:045fedcfadf6
    74   unfolding fun_eq_iff
    74   unfolding fun_eq_iff
    75   by (simp add: Quotient_abs_rep[OF set_quotient[OF assms]])
    75   by (simp add: Quotient_abs_rep[OF set_quotient[OF assms]])
    76 
    76 
    77 lemma mem_prs[quot_preserve]:
    77 lemma mem_prs[quot_preserve]:
    78   assumes "Quotient R Abs Rep"
    78   assumes "Quotient R Abs Rep"
       
    79   shows "(Rep ---> (Abs ---> id) ---> id) (op \<in>) = op \<in>"
       
    80 using Quotient_abs_rep[OF assms]
       
    81 by(simp add: fun_eq_iff mem_def)
       
    82 
       
    83 lemma mem_rsp[quot_respect]:
       
    84   "(R ===> (R ===> op =) ===> op =) (op \<in>) (op \<in>)"
       
    85   by (auto simp add: fun_eq_iff mem_def intro!: fun_relI elim: fun_relE)
       
    86 
       
    87 lemma mem_prs2:
       
    88   assumes "Quotient R Abs Rep"
    79   shows "(Rep ---> op -` Abs ---> id) op \<in> = op \<in>"
    89   shows "(Rep ---> op -` Abs ---> id) op \<in> = op \<in>"
    80   by (simp add: fun_eq_iff Quotient_abs_rep[OF assms])
    90   by (simp add: fun_eq_iff Quotient_abs_rep[OF assms])
    81 
    91 
    82 lemma mem_rsp[quot_respect]:
    92 lemma mem_rsp2:
    83   shows "(R ===> set_rel R ===> op =) op \<in> op \<in>"
    93   shows "(R ===> set_rel R ===> op =) op \<in> op \<in>"
    84   by (intro fun_relI) (simp add: set_rel_def)
    94   by (intro fun_relI) (simp add: set_rel_def)
    85 
    95 
    86 end
    96 end