src/HOL/Library/Quotient_List.thy
changeset 63649 e690d6f2185b
parent 62954 c5d0fdc260fa
child 67399 eab6ce8368fa
--- a/src/HOL/Library/Quotient_List.thy	Wed Aug 10 09:33:54 2016 +0200
+++ b/src/HOL/Library/Quotient_List.thy	Wed Aug 10 14:50:59 2016 +0200
@@ -145,7 +145,6 @@
   shows "((abs1 ---> abs2 ---> rep1) ---> rep1 ---> (map rep2) ---> abs1) foldl = foldl"
   by (simp add: fun_eq_iff foldl_prs_aux [OF a b])
 
-(* induct_tac doesn't accept 'arbitrary', so we manually 'spec' *)
 lemma foldl_rsp[quot_respect]:
   assumes q1: "Quotient3 R1 Abs1 Rep1"
   and     q2: "Quotient3 R2 Abs2 Rep2"