changeset 47351 | 0193e663a19e |
parent 47325 | ec6187036495 |
child 47354 | 95846613e414 |
--- a/src/HOL/Lifting.thy Wed Apr 04 13:41:38 2012 +0200 +++ b/src/HOL/Lifting.thy Wed Apr 04 13:42:01 2012 +0200 @@ -273,6 +273,11 @@ show "transp (invariant P)" by (auto intro: transpI simp: invariant_def) qed +lemma Quotient_to_transfer: + assumes "Quotient R Abs Rep T" and "R c c" and "c' \<equiv> Abs c" + shows "T c c'" + using assms by (auto dest: Quotient_cr_rel) + subsection {* ML setup *} text {* Auxiliary data for the lifting package *}