Edited Unassigned: Auto-triggers on set, iset, map, and imap [151]
Currently, when one uses a set comprehension, Dafny doesn't automatically put a trigger on the corresponding existential. You can override this behavior with {:trigger}, but it would be nice if Dafny...
View ArticleCreated 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?
View ArticleNew Post: getting counterexamples
Is it possible to get counterexamples from the web interface? I am having trouble realizing why the following code does not check out:class KV { var key : int; var value : int; constructor (k: int, v:...
View ArticleNew Post: possible bug?
For this code:function method sum (s: seq<int>) : int { if |s| == 0 then 0 else s[0] + sum(s[1..]) } class KV { var key : int; var value : int; predicate equals (o: KV) reads this, o requires o...
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: It is something to do with having arithmetic operations in...
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: Here is a `calc` version: http://rise4fun.com/Dafny/6UNv ```...
View ArticleNew Post: possible bug?
I think input == v2 is an intermediate assertion to infer v3 == sum(input). the postconditions fromvar v1 := mapper(input); var v2,v3 := reduce(v1); are:v1 is a sequence of KV which is generated based...
View ArticleNew Post: Express relations and their properties
Hello: I want to represent some relations in Dafny and state that they follow certain properties like transitivity, antisymmetry or totalness. For example, suppose we want to declare a binary relation...
View ArticleSource code checked in, #c90e0803674e
Add fuel synonym that allow Z3 to go from any fuel constants to LZ. This includes: -- defining a new Boogie-level un-interpreted function, named "IsFuelBottom" from type Layer to Layer. -- Add assume...
View ArticleNew Post: Express relations and their properties
I don't see immediately how you can do this. You need to prove that the predicate is defined. The terminiation error means that Dafny can't prove it is defined. Here are some random thoughts: To show...
View ArticleNew Post: Express relations and their properties
One option would be to write your predicate without any ensures initially, write a lemma ensuring its properties, and then write a wrapper around the original predicate. It can provide ensures about...
View ArticleSource code checked in, #0861864d05bc
Fix issue 155. Allow multiset of objects in the reads clause.
View Article