diff -r 44fa9df44e6f -r 57073b0b8fac IntEx.thy --- a/IntEx.thy Fri Dec 04 15:41:09 2009 +0100 +++ b/IntEx.thy Fri Dec 04 15:50:57 2009 +0100 @@ -1,7 +1,6 @@ theory IntEx imports QuotMain begin - fun intrel :: "(nat \ nat) \ (nat \ nat) \ bool" (infix "\" 50) @@ -237,12 +236,12 @@ by (simp_all add: Quotient_ABS_REP[OF a]) lemma cons_rsp[quotient_rsp]: - "(op \ ===> LIST_REL op \ ===> LIST_REL op \) op # op #" + "(op \ ===> list_rel op \ ===> list_rel op \) op # op #" by simp (* I believe it's true. *) lemma foldl_rsp[quotient_rsp]: - "((op \ ===> op \ ===> op \) ===> op \ ===> LIST_REL op \ ===> op \) foldl foldl" + "((op \ ===> op \ ===> op \) ===> op \ ===> list_rel op \ ===> op \) foldl foldl" apply (simp only: fun_rel.simps) apply (rule allI) apply (rule allI) @@ -257,7 +256,7 @@ sorry lemma nil_listrel_rsp[quotient_rsp]: - "(LIST_REL R) [] []" + "(list_rel R) [] []" by simp lemma "foldl PLUS x [] = x"