author | paulson |
Tue, 05 Apr 2005 13:05:20 +0200 | |
changeset 15655 | 157f3988f775 |
parent 15654 | d53e5370cfbf |
child 15656 | 988f91b9c4ef |
src/HOL/HOL.thy | file | annotate | diff | comparison | revisions |
--- a/src/HOL/HOL.thy Tue Apr 05 08:03:52 2005 +0200 +++ b/src/HOL/HOL.thy Tue Apr 05 13:05:20 2005 +0200 @@ -270,6 +270,12 @@ apply (rule refl) done +lemma arg_cong2: "\<lbrakk> a = b; c = d \<rbrakk> \<Longrightarrow> f a c = f b d" +apply (erule ssubst)+ +apply (rule refl) +done + + lemma cong: "[| f = g; (x::'a) = y |] ==> f(x) = g(y)" apply (erule subst)+ apply (rule refl)