changeset 71954 | 13bb3f5cdc5b |
parent 70185 | ac1706cdde25 |
child 72488 | ee659bca8955 |
--- a/src/HOL/SPARK/SPARK.thy Thu Jun 18 09:07:30 2020 +0000 +++ b/src/HOL/SPARK/SPARK.thy Thu Jun 18 09:07:30 2020 +0000 @@ -37,7 +37,7 @@ XOR_upper [of _ 64, simplified] lemma bit_not_spark_eq: - "NOT (word_of_int x :: ('a::len0) word) = + "NOT (word_of_int x :: ('a::len) word) = word_of_int (2 ^ LENGTH('a) - 1 - x)" proof - have "word_of_int x + NOT (word_of_int x) =