Edited Unassigned: Dafny verifies incorrect assertions [145]
Consider the following code fragment ([http://rise4fun.com/Dafny/6lkz](http://rise4fun.com/Dafny/6lkz)):```function existential(mat: array2<bool>): bool requires mat != null{ exists i, j :: 0...
View ArticleCommented Unassigned: Dafny verifies incorrect assertions [145]
Consider the following code fragment ([http://rise4fun.com/Dafny/6lkz](http://rise4fun.com/Dafny/6lkz)):```function existential(mat: array2<bool>): bool requires mat != null{ exists i, j :: 0...
View ArticleClosed Unassigned: Dafny verifies incorrect assertions [145]
Consider the following code fragment ([http://rise4fun.com/Dafny/6lkz](http://rise4fun.com/Dafny/6lkz)):```function existential(mat: array2<bool>): bool requires mat != null{ exists i, j :: 0...
View ArticleSource code checked in, #8c65861d2c97
Fix issue 146. Add check for insufficient reads clause to read array elements.
View ArticleEdited Unassigned: Dafny verifies incorrect assertions (updated) [146]
I cloned and built the latest version of Dafny (changeset d954a409627e), found happily that #145 is fixed, and proceeded with my project. Unfortunately, I soon encountered another bug, similar to the...
View ArticleCommented Unassigned: Dafny verifies incorrect assertions (updated) [146]
I cloned and built the latest version of Dafny (changeset d954a409627e), found happily that #145 is fixed, and proceeded with my project. Unfortunately, I soon encountered another bug, similar to the...
View ArticleClosed Unassigned: Dafny verifies incorrect assertions (updated) [146]
I cloned and built the latest version of Dafny (changeset d954a409627e), found happily that #145 is fixed, and proceeded with my project. Unfortunately, I soon encountered another bug, similar to the...
View ArticleSource code checked in, #3918cfb0b419
Test cases with nested lambdas. There's much room for improvement.
View ArticleCommented Unassigned: A timed out [157]
Please, have a look to the lemma proof:http://rise4fun.com/Dafny/jeadI cannot think what is the problem there!!!Some help, please?Comments: Thank you for the previous explanations and sorry for the...
View ArticleCommented Unassigned: A timed out [157]
Please, have a look to the lemma proof:http://rise4fun.com/Dafny/jeadI cannot think what is the problem there!!!Some help, please?Comments: Moreover, Dafny fails also to prove the assertion with the...
View ArticleCommented Unassigned: A timed out [157]
Please, have a look to the lemma proof:http://rise4fun.com/Dafny/jeadI cannot think what is the problem there!!!Some help, please?Comments: Also related is that the following lemma Sum_Prod_Lemma is...
View ArticleCreated Unassigned: Generic type equality for datatypes with iset and imap [162]
The example below gives errors about type equality in the A and C cases, but not the B or D cases, nor in the cases that don't use datatypes, which suggests there's a datatype-related code path that's...
View ArticleEdited Unassigned: Var such-that for non-primitive types [161]
The following should verify, but fails. If t is changed to "int", it does verify. This seems to have something to do with the treatment of :| for non-primitive types like seq<int>.```type t =...
View ArticleClosed Unassigned: Var such-that for non-primitive types [161]
The following should verify, but fails. If t is changed to "int", it does verify. This seems to have something to do with the treatment of :| for non-primitive types like seq<int>.```type t =...
View ArticleEdited Unassigned: Generic type equality for datatypes with iset and imap [162]
The example below gives errors about type equality in the A and C cases, but not the B or D cases, nor in the cases that don't use datatypes, which suggests there's a datatype-related code path that's...
View ArticleClosed Unassigned: Generic type equality for datatypes with iset and imap [162]
The example below gives errors about type equality in the A and C cases, but not the B or D cases, nor in the cases that don't use datatypes, which suggests there's a datatype-related code path that's...
View ArticleCommented Unassigned: Generic type equality for datatypes with iset and imap...
The example below gives errors about type equality in the A and C cases, but not the B or D cases, nor in the cases that don't use datatypes, which suggests there's a datatype-related code path that's...
View ArticleSource code checked in, #39d0dcc4247c
Fix issue 161. Add $Is and $IsAlloc for the $let$_canCall axiom. So for let-such-that expression: var x:X, y:Y :| P(x,y,g); F(...) the axiom will be axiom (forall g:G :: { $let$x(g) } { $let$y(g) }...
View ArticleSource code checked in, #24ffff36b7d5
Fix issue 162. IndDatatype of iMap and iSet was mistakenly marked as never support equality.
View Article