src/HOL/SMT_Examples/SMT_Word_Examples.thy
changeset 58410 6d46ad54a2ab
parent 58367 8af1e68d7e1a
child 58889 5b7a9633cfa8
--- a/src/HOL/SMT_Examples/SMT_Word_Examples.thy	Sun Sep 21 16:56:06 2014 +0200
+++ b/src/HOL/SMT_Examples/SMT_Word_Examples.thy	Sun Sep 21 16:56:11 2014 +0200
@@ -27,7 +27,7 @@
 lemma "27 + 11 = (6::5 word)" by smt
 lemma "7 * 3 = (21::8 word)" by smt
 lemma "11 - 27 = (-16::8 word)" by smt
-lemma "- -11 = (11::5 word)" by smt
+lemma "- (- 11) = (11::5 word)" by smt
 lemma "-40 + 1 = (-39::7 word)" by smt
 lemma "a + 2 * b + c - b = (b + c) + (a :: 32 word)" by smt
 lemma "x = (5 :: 4 word) \<Longrightarrow> 4 * x = 4" by smt