Skip to content
Snippets Groups Projects
Commit 7ff0e1c1 authored by Patrick Baudin's avatar Patrick Baudin
Browse files

Merge branch 'feature/patrick/wp-list-simplification' into 'master'

[WP] minor changes in tests

See merge request frama-c/frama-c!3559
parents 2a1f5d79 6c0a3a08
No related branches found
No related tags found
No related merge requests found
...@@ -40,7 +40,7 @@ ...@@ -40,7 +40,7 @@
check lemma not_nil_elt: ok: ([| 1 |] ^ A) != A ; check lemma not_nil_elt: ok: ([| 1 |] ^ A) != A ;
check lemma repeat1: ko: (S *^ N) == (S *^ M) check lemma repeat1: ok: (S *^ N) == (S *^ M)
<==> ( N == M || ( ((S *^ N) ^ A) == A && ((S *^ M) ^ A) == A ) ) ; <==> ( N == M || ( ((S *^ N) ^ A) == A && ((S *^ M) ^ A) == A ) ) ;
check lemma repeat2: ok: ( ((S *^ N) ^ S) *^ M ) == ( ( S ^ (S *^ N)) *^ M ) ; check lemma repeat2: ok: ( ((S *^ N) ^ S) *^ M ) == ( ( S ^ (S *^ N)) *^ M ) ;
...@@ -50,9 +50,9 @@ ...@@ -50,9 +50,9 @@
check lemma left_unfold_repeat1: ok: ( ((S ^ A ^ B) *^ 3) ^ A ^ S ) == (S ^ C) check lemma left_unfold_repeat1: ok: ( ((S ^ A ^ B) *^ 3) ^ A ^ S ) == (S ^ C)
<==> ( A ^ B ^ ((S ^ A ^ B) *^ 2) ^ A ^ S ) == ( C); <==> ( A ^ B ^ ((S ^ A ^ B) *^ 2) ^ A ^ S ) == ( C);
check lemma right_shift_repeat1: ko: ( A ^ S ^ ((B ^ A ^ S) *^ N) ) == (C ^ S) check lemma right_shift_repeat1: ok: ( A ^ S ^ ((B ^ A ^ S) *^ N) ) == (C ^ S)
<==> ( A ^ ((S ^ B ^ A ) *^ N) ) == (C ); <==> ( A ^ ((S ^ B ^ A ) *^ N) ) == (C );
check lemma right_unfold_repeat1: ko: ( S ^ A ^ ((B ^ A ^ S) *^ 3) ) == (C ^ S) check lemma right_unfold_repeat1: ok: ( S ^ A ^ ((B ^ A ^ S) *^ 3) ) == (C ^ S)
<==> ( S ^ A ^ ((B ^ A ^ S) *^ 2) ^ B ^ A) == (C ); <==> ( S ^ A ^ ((B ^ A ^ S) *^ 2) ^ B ^ A) == (C );
...@@ -61,13 +61,13 @@ ...@@ -61,13 +61,13 @@
check lemma left_unfold_repeat2: ok: ( ((S ^ A ^ B) *^ 3) ^ C) == (S ^ A) check lemma left_unfold_repeat2: ok: ( ((S ^ A ^ B) *^ 3) ^ C) == (S ^ A)
<==> (A ^ A ^ B ^ C ^ S) == A ; <==> (A ^ A ^ B ^ C ^ S) == A ;
check lemma right_shift_repeat2: ko: ( C ^ A ^ S ^ ((B ^ A ^ S) *^ N) ) == (A ^ S) check lemma right_shift_repeat2: ok: ( C ^ A ^ S ^ ((B ^ A ^ S) *^ N) ) == (A ^ S)
<==> ( (C ^ S) == S && (N<=0 || (A ^ B ^ S ^ S) == S) ); <==> ( (C ^ S) == S && (N<=0 || (A ^ B ^ S ^ S) == S) );
check lemma right_unfold_repeat2: ko: ( C ^ ((B ^ A ^ S) *^ 3) ) == (A ^ S) check lemma right_unfold_repeat2: ok: ( C ^ ((B ^ A ^ S) *^ 3) ) == (A ^ S)
<==> (A ^ B ^ C ^ S ^ S) == S ; <==> (A ^ B ^ C ^ S ^ S) == S ;
check lemma subsequence1: ko: ( A ^ (S *^ N) ^ B ^ S ^ C ) == ( (S *^ N) ^ S ) check lemma subsequence1: ok: ( A ^ (S *^ N) ^ B ^ S ^ C ) == ( (S *^ N) ^ S )
<==> ( A ^ B ^ C ^ C ) == C ; <==> ( A ^ B ^ C ^ C ) == C ;
} }
......
...@@ -18,16 +18,16 @@ ...@@ -18,16 +18,16 @@
[wp] [Qed] Goal typed_check_lemma_nth_repeat_3_ok : Valid [wp] [Qed] Goal typed_check_lemma_nth_repeat_3_ok : Valid
[wp] [Qed] Goal typed_check_lemma_nth_repeat_4_ok : Valid [wp] [Qed] Goal typed_check_lemma_nth_repeat_4_ok : Valid
[wp] [Alt-Ergo] Goal typed_check_lemma_nth_repeat_undefined_1_ko : Unsuccess [wp] [Alt-Ergo] Goal typed_check_lemma_nth_repeat_undefined_1_ko : Unsuccess
[wp] [Qed] Goal typed_check_lemma_repeat1_ko : Valid [wp] [Qed] Goal typed_check_lemma_repeat1_ok : Valid
[wp] [Qed] Goal typed_check_lemma_repeat2_ok : Valid [wp] [Qed] Goal typed_check_lemma_repeat2_ok : Valid
[wp] [Qed] Goal typed_check_lemma_repeat_nil_ok : Valid [wp] [Qed] Goal typed_check_lemma_repeat_nil_ok : Valid
[wp] [Qed] Goal typed_check_lemma_repeat_one_ok : Valid [wp] [Qed] Goal typed_check_lemma_repeat_one_ok : Valid
[wp] [Qed] Goal typed_check_lemma_repeat_repeated_ok : Valid [wp] [Qed] Goal typed_check_lemma_repeat_repeated_ok : Valid
[wp] [Qed] Goal typed_check_lemma_right_shift_repeat1_ko : Valid [wp] [Qed] Goal typed_check_lemma_right_shift_repeat1_ok : Valid
[wp] [Qed] Goal typed_check_lemma_right_shift_repeat2_ko : Valid [wp] [Qed] Goal typed_check_lemma_right_shift_repeat2_ok : Valid
[wp] [Qed] Goal typed_check_lemma_right_unfold_repeat1_ko : Valid [wp] [Qed] Goal typed_check_lemma_right_unfold_repeat1_ok : Valid
[wp] [Qed] Goal typed_check_lemma_right_unfold_repeat2_ko : Valid [wp] [Qed] Goal typed_check_lemma_right_unfold_repeat2_ok : Valid
[wp] [Qed] Goal typed_check_lemma_subsequence1_ko : Valid [wp] [Qed] Goal typed_check_lemma_subsequence1_ok : Valid
[wp] Proved goals: 25 / 26 [wp] Proved goals: 25 / 26
Qed: 22 Qed: 22
Alt-Ergo: 3 (unsuccess: 1) Alt-Ergo: 3 (unsuccess: 1)
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment