diff -r cc1f240d8cf4 -r fdfeef0399f7 QuotMain.thy --- a/QuotMain.thy Fri Dec 04 11:34:21 2009 +0100 +++ b/QuotMain.thy Fri Dec 04 11:34:49 2009 +0100 @@ -136,16 +136,6 @@ end -(* EQUALS_RSP is stronger *) -lemma equiv_trans2: - assumes e: "EQUIV R" - and ac: "R a c" - and bd: "R b d" - shows "R a b = R c d" -using ac bd e -unfolding EQUIV_REFL_SYM_TRANS TRANS_def SYM_def -by (blast) - section {* type definition for the quotient type *} (* the auxiliary data for the quotient types *) @@ -1343,7 +1333,8 @@ val rthm' = atomize_thm rthm val rule = procedure_inst context (prop_of rthm') (term_of concl) val rel_refl = map (fn x => @{thm EQUIV_REFL} OF [x]) rel_eqv - val trans2 = map (fn x => @{thm equiv_trans2} OF [x]) rel_eqv + val quotients = quotient_rules_get lthy + val trans2 = map (fn x => @{thm EQUALS_RSP} OF [x]) quotients val thm = Drule.instantiate' [] [SOME (snd (Thm.dest_comb concl))] @{thm QUOT_TRUE_i} in EVERY1