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

[WP] adds one more test

parent 30345328
No related branches found
No related tags found
No related merge requests found
...@@ -57,7 +57,8 @@ ...@@ -57,7 +57,8 @@
<==> (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 )
<==> ( A ^ B ^ C ^ C ) == C ;
} }
*/ */
......
...@@ -51,6 +51,11 @@ Prove: let a_0 = (concat L_B L_A L_S) in ...@@ -51,6 +51,11 @@ Prove: let a_0 = (concat L_B L_A L_S) in
Lemma right_unfold_repeat2: Lemma right_unfold_repeat2:
Prove: true Prove: true
------------------------------------------------------------
Lemma subsequence1:
Prove: true
------------------------------------------------------------ ------------------------------------------------------------
------------------------------------------------------------ ------------------------------------------------------------
Axiomatic 'MkRepeat' Axiomatic 'MkRepeat'
......
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