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] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- Subject: [Frama-c-discuss] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- From: pmsf at lia.ufc.br (Pablo M. S. Farias)
- Date: Tue, 08 Mar 2016 15:19:39 -0300
- In-reply-to: <76ca8494dbcab197d69051a37cdc73bc@lia.ufc.br>
- References: <76ca8494dbcab197d69051a37cdc73bc@lia.ufc.br>
Just to say that the compatibility between WP 0.9 and Coq 8.5 is not urgent for me anymore: I created a fresh opam environment with Coq 8.4pl6 + Why3 + Frama-C. (I still cannot verify the lemma, though.) --- Pablo http://lia.ufc.br/~pmsf/ Em 2016-03-08 13:22, Pablo M. S. Farias escreveu: > Hello, all! > > As reported in the previous e-mail, I'm having trouble verifying this > in WP (also attached): > > /*@ lemma ptr_inc: \forall int n, *v, *p; > n >= 0 ==> \valid_read(v + (0..n-1)) ==> v <= p < v+n ==> > v <= p+1; > */ > > I would like to use Coq to try out a proof, but running > > frama-c-gui -wp -wp-prover coqide lemma_ptr_inc.c > > gives this output: > > [kernel] Parsing FRAMAC_SHARE/libc/__fc_builtin_for_normalization.i > (no preprocessing) > [kernel] Parsing lemma_ptr_inc.c (with preprocessing) > [wp] Running WP plugin... > [wp] Collecting axiomatic usage > [wp] 1 goal scheduled > [wp] [Coq] Compiling 'BuiltIn.v'. > [wp] [Coq] 'BuiltIn.v' compilation failed. > Don't know what to do with -as bool -as int -as real -as map > See -help for the list of supported options > [wp] [Coq] Goal typed_lemma_ptr_inc : Failed > Error: Compilation of 'BuiltIn.v' failed. > [wp] Proved goals: 0 / 1 > Coq: 0 (failed: 1) > > Is WP 0.9 (for Magnesium-20151002) compatible with Coq 8.5 (which I'm > using)? Am I doing something wrong? > > Thanks in advance, > > -- > Pablo > http://lia.ufc.br/~pmsf/
- Follow-Ups:
- [Frama-c-discuss] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- From: Patrick.Baudin at cea.fr (BAUDIN Patrick)
- [Frama-c-discuss] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- References:
- [Frama-c-discuss] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- From: pmsf at lia.ufc.br (Pablo M. S. Farias)
- [Frama-c-discuss] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- Prev by Date: [Frama-c-discuss] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- Next by Date: [Frama-c-discuss] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- Previous by thread: [Frama-c-discuss] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- Next by thread: [Frama-c-discuss] WP 0.9 (for Magnesium) Compatible with Coq 8.5?
- Index(es):