Frama-C-discuss mailing list archives
This page gathers the archives of the old Frama-C-discuss archives, that was hosted by Inria's gforge before its demise at the end of 2020. To search for mails newer than September 2020, please visit the page of the new mailing list on Renater.
[Date Prev][Date Next][Thread Prev][Thread Next][Date Index][Thread Index]
[Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- Subject: [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- From: loic.correnson at cea.fr (Loïc Correnson)
- Date: Mon, 9 May 2016 10:21:05 +0200
- In-reply-to: <572D7FCB.8000007@inria.fr>
- References: <4086A395-805E-41FD-8B38-060121C33B8D@cea.fr> <1838053228.5811460.1462368437087.JavaMail.yahoo@mail.yahoo.com> <7D60673F-361D-4DCD-A207-D883487FAFBD@cea.fr> <572D7FCB.8000007@inria.fr>
> Just a guess : if you write 2.0 and 1.0 instead of 2 and 1 does it work? > If yes, then it is an issue with conversion from integer to real. No it is not. The generated lemma for Why3 is: (* ---------------------------------------------------------- *) (* --- Global Definitions --- *) (* ---------------------------------------------------------- *) theory Axiomatic use import bool.Bool use import int.Int use import int.ComputerDivision use import real.RealInfix use import Qed.Qed use import int.Abs as IAbs use import map.Map lemma Q_POS: forall x : real. (2.0e0 *. x) <=. (1.0e0 +. (x *. x)) end None of CVC4, Z3 and Alt-Ergo is able to prove it â but in Coq it is. L.
- References:
- [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- From: loic.correnson at cea.fr (Loïc Correnson)
- [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- From: cok at frontiernet.net (cok at frontiernet.net)
- [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- From: loic.correnson at cea.fr (Loïc Correnson)
- [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- From: Claude.Marche at inria.fr (Claude Marché)
- [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- Prev by Date: [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- Next by Date: [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- Previous by thread: [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- Next by thread: [Frama-c-discuss] hint assertions and understanding cooperation between wp and value plugin
- Index(es):