diff -r 173667d73115 -r 4eb98849c5c0 src/HOL/SMT_Examples/SMT_Tests.thy --- a/src/HOL/SMT_Examples/SMT_Tests.thy Mon Jul 12 22:35:41 2010 +0200 +++ b/src/HOL/SMT_Examples/SMT_Tests.thy Tue Jul 13 02:29:05 2010 +0200 @@ -84,6 +84,7 @@ lemma "case P of True \ P | False \ \P" + "case P of False \ \P | True \ P" "case \P of True \ \P | False \ P" "case P of True \ (Q \ P) | False \ (P \ Q)" by smt+ @@ -176,6 +177,11 @@ by smt+ lemma + "(\x\M. P x) \ c \ M \ P c" + "(\x\M. P x) \ \(P c \ c \ M)" + by smt+ + +lemma "let P = True in P" "let P = P1 \ P2 in P \ \P" "let P1 = True; P2 = False in P1 \ P2 \ P2 \ P1"