diff -r 70deefb6c093 -r 8f10b0e77d94 src/HOL/SMT/Examples/SMT_Examples.thy --- a/src/HOL/SMT/Examples/SMT_Examples.thy Wed Apr 07 19:48:58 2010 +0200 +++ b/src/HOL/SMT/Examples/SMT_Examples.thy Wed Apr 07 20:38:11 2010 +0200 @@ -539,7 +539,8 @@ lemma "i \ i1 \ i \ i2 \ (f (i1 := v1, i2 := v2)) i = f i" by smt -lemma "(f g x = (g x \ True)) \ (f g x = True) \ (g x = True)" by smt +lemma "(f g (x::'a::type) = (g x \ True)) \ (f g x = True) \ (g x = True)" + by smt lemma "id 3 = 3 \ id True = True" by (smt id_def)