是否可以对 ACSL 中定义的归纳谓词使用归纳?
考虑ACSL 手册中的以下示例:
struct List {
int value;
struct List* next;
};
/*@ inductive reachable{L}(struct List* root, struct List* to) {
@ case empty{L}: \forall struct List* l; reachable(l, l);
@ case non_empty{L}: \forall struct List *l1,*l2;
@ \valid(l1) && reachable(l1->next, l2) ==> reachable(l1, l2);
@ }
*/
我试图证明以下引理:
/*@ lemma next_null_reachable: \forall struct List* l;
@ \valid(l) && reachable(l, \null) ==> reachable(l->next, \null);
*/
Alt-Ergo 在这里失败了,所以我求助于手动 Coq 推理:
Goal
forall (t : array Z),
forall (t_1 : farray addr addr),
forall (a : addr),
((valid_rw t a 2%Z)) ->
((P_reachable t t_1 a (null))) ->
((P_reachable t t_1 (t_1.[ (shiftfield_F_List_next a) ]) (null))).
但是当 I 时Search P_reachable
,我发现只生成了两个公理:
Q_non_empty:
forall (t : array int) (t_1 : farray addr addr) (a_1 a : addr),
valid_rw t a_1 2 ->
P_reachable t t_1 (t_1 .[ shiftfield_F_List_next a_1]) a ->
P_reachable t t_1 a_1 a
Q_empty:
forall (t : array int) (t_1 : farray addr addr) (a : addr),
P_reachable t t_1 a a
并且没有感应原理。所以我不能申请induction P_reachable
或destruct P_reachable
。
我使用frama-c
版本 Sodium-20150201 的 WP 插件。
要重现,您可以运行frama-c -wp -wp-rte -wp-prover coqide file.c
,其中file.c
包含List
和reachable
定义和next_null_reachable
引理。