Quot/QuotList.thy
changeset 796 64f9c76f70c7
parent 768 e9e205b904e2
child 825 970e86082cd7
--- a/Quot/QuotList.thy	Sat Dec 26 21:36:20 2009 +0100
+++ b/Quot/QuotList.thy	Sat Dec 26 23:20:46 2009 +0100
@@ -125,7 +125,7 @@
   shows "abs2 (foldr ((abs1 ---> abs2 ---> rep2) f) (map rep1 l) (rep2 e)) = foldr f l e"
 by (induct l) (simp_all add: Quotient_abs_rep[OF a] Quotient_abs_rep[OF b])
 
-lemma foldr_prs[quot_respect]:
+lemma foldr_prs[quot_preserve]:
   assumes a: "Quotient R1 abs1 rep1"
   and     b: "Quotient R2 abs2 rep2"
   shows "((abs1 ---> abs2 ---> rep2) ---> (map rep1) ---> rep2 ---> abs2) foldr = foldr"