1/-1 %// 2 cases not validating or computing #2913
-
Folks, open FStar.Math let lemma_zero_div_two (i: int{i = 0}) : Lemma (i / 2 = 0) = () let lemma_one_div_two (i: int{i = 1}) : Lemma (i / 2 = 0) = () [@@ expect_failure] [@@ expect_failure] [@@ expect_failure] |
Beta Was this translation helpful? Give feedback.
Replies: 2 comments
-
let lemma_minus_one_div_two' = assert((-1) / 2 = -1) is worse, bug submitted. |
Beta Was this translation helpful? Give feedback.
-
Nik says that this is Euclidean arithmetic and should be the answer to all above. |
Beta Was this translation helpful? Give feedback.
Nik says that this is Euclidean arithmetic and should be the answer to all above.
Testing this, it's right. Odd but right.