src/HOL/Lifting.thy
changeset 71262 a30278c8585f
parent 69913 ca515cf61651
equal deleted inserted replaced
71261:4765fec43414 71262:a30278c8585f
   543 by (simp add: eq_onp_def Domainp_iff[abs_def] Quotient_cr_rel[OF assms])
   543 by (simp add: eq_onp_def Domainp_iff[abs_def] Quotient_cr_rel[OF assms])
   544 
   544 
   545 end
   545 end
   546 
   546 
   547 (* needed for lifting_def_code_dt.ML (moved from Lifting_Set) *)
   547 (* needed for lifting_def_code_dt.ML (moved from Lifting_Set) *)
   548 lemma right_total_UNIV_transfer: 
   548 lemma right_total_UNIV_transfer:
   549   assumes "right_total A"
   549   assumes "right_total A"
   550   shows "(rel_set A) (Collect (Domainp A)) UNIV"
   550   shows "(rel_set A) (Collect (Domainp A)) UNIV"
   551   using assms unfolding right_total_def rel_set_def Domainp_iff by blast
   551   using assms unfolding right_total_def rel_set_def Domainp_iff by blast
   552 
   552 
   553 subsection \<open>ML setup\<close>
   553 subsection \<open>ML setup\<close>