src/HOL/Lifting.thy
changeset 67229 4ecf0ef70efb
parent 63343 fb5d8a50c641
child 67399 eab6ce8368fa
equal deleted inserted replaced
67228:7c7b76695c90 67229:4ecf0ef70efb
   226 
   226 
   227 lemma UNIV_typedef_to_equivp:
   227 lemma UNIV_typedef_to_equivp:
   228   fixes Abs :: "'a \<Rightarrow> 'b"
   228   fixes Abs :: "'a \<Rightarrow> 'b"
   229   and Rep :: "'b \<Rightarrow> 'a"
   229   and Rep :: "'b \<Rightarrow> 'a"
   230   assumes "type_definition Rep Abs (UNIV::'a set)"
   230   assumes "type_definition Rep Abs (UNIV::'a set)"
   231   shows "equivp (op=::'a\<Rightarrow>'a\<Rightarrow>bool)"
   231   shows "equivp (op= ::'a\<Rightarrow>'a\<Rightarrow>bool)"
   232 by (rule identity_equivp)
   232 by (rule identity_equivp)
   233 
   233 
   234 lemma typedef_to_Quotient:
   234 lemma typedef_to_Quotient:
   235   assumes "type_definition Rep Abs S"
   235   assumes "type_definition Rep Abs S"
   236   and T_def: "T \<equiv> (\<lambda>x y. x = Rep y)"
   236   and T_def: "T \<equiv> (\<lambda>x y. x = Rep y)"