Datasets:
Tasks:
Text Generation
Modalities:
Text
Sub-tasks:
language-modeling
Languages:
English
Size:
100K - 1M
License:
theory ASC_Sufficiency | |
imports ASC_Suite | |
begin | |
section \<open> Sufficiency of the test suite to test for reduction \<close> | |
text \<open> | |
This section provides a proof that the test suite generated by the adaptive state counting algorithm | |
is sufficient to test for reduction. | |
\<close> | |
subsection \<open> Properties of minimal sequences to failures extending the deterministic state cover \<close> | |
text \<open> | |
The following two lemmata show that minimal sequences to failures extending the deterministic state | |
cover do not with their extending suffix visit any state twice or visit a state also reached by a | |
sequence in the chosen permutation of reactions to the deterministic state cover. | |
\<close> | |
lemma minimal_sequence_to_failure_extending_implies_Rep_Pre : | |
assumes "minimal_sequence_to_failure_extending V M1 M2 vs xs" | |
and "OFSM M1" | |
and "OFSM M2" | |
and "test_tools M2 M1 FAIL PM V \<Omega>" | |
and "V'' \<in> N (vs@xs') M1 V" | |
and "prefix xs' xs" | |
shows "\<not> Rep_Pre M2 M1 vs xs'" | |
proof | |
assume "Rep_Pre M2 M1 vs xs'" | |
then obtain xs1 xs2 s1 s2 where "prefix xs1 xs2" | |
"prefix xs2 xs'" | |
"xs1 \<noteq> xs2" | |
"io_targets M2 (initial M2) (vs @ xs1) = {s2}" | |
"io_targets M2 (initial M2) (vs @ xs2) = {s2}" | |
"io_targets M1 (initial M1) (vs @ xs1) = {s1}" | |
"io_targets M1 (initial M1) (vs @ xs2) = {s1}" | |
by auto | |
then have "s2 \<in> io_targets M2 (initial M2) (vs @ xs1)" | |
"s2 \<in> io_targets M2 (initial M2) (vs @ xs2)" | |
"s1 \<in> io_targets M1 (initial M1) (vs @ xs1)" | |
"s1 \<in> io_targets M1 (initial M1) (vs @ xs2)" | |
by auto | |
have "vs@xs1 \<in> L M1" | |
using io_target_implies_L[OF \<open>s1 \<in> io_targets M1 (initial M1) (vs @ xs1)\<close>] by assumption | |
have "vs@xs2 \<in> L M1" | |
using io_target_implies_L[OF \<open>s1 \<in> io_targets M1 (initial M1) (vs @ xs2)\<close>] by assumption | |
have "vs@xs1 \<in> L M2" | |
using io_target_implies_L[OF \<open>s2 \<in> io_targets M2 (initial M2) (vs @ xs1)\<close>] by assumption | |
have "vs@xs2 \<in> L M2" | |
using io_target_implies_L[OF \<open>s2 \<in> io_targets M2 (initial M2) (vs @ xs2)\<close>] by assumption | |
obtain tr1_1 where "path M1 (vs@xs1 || tr1_1) (initial M1)" | |
"length tr1_1 = length (vs@xs1)" | |
"target (vs@xs1 || tr1_1) (initial M1) = s1" | |
using \<open>s1 \<in> io_targets M1 (initial M1) (vs @ xs1)\<close> by auto | |
obtain tr1_2 where "path M1 (vs@xs2 || tr1_2) (initial M1)" | |
"length tr1_2 = length (vs@xs2)" | |
"target (vs@xs2 || tr1_2) (initial M1) = s1" | |
using \<open>s1 \<in> io_targets M1 (initial M1) (vs @ xs2)\<close> by auto | |
obtain tr2_1 where "path M2 (vs@xs1 || tr2_1) (initial M2)" | |
"length tr2_1 = length (vs@xs1)" | |
"target (vs@xs1 || tr2_1) (initial M2) = s2" | |
using \<open>s2 \<in> io_targets M2 (initial M2) (vs @ xs1)\<close> by auto | |
obtain tr2_2 where "path M2 (vs@xs2 || tr2_2) (initial M2)" | |
"length tr2_2 = length (vs@xs2)" | |
"target (vs@xs2 || tr2_2) (initial M2) = s2" | |
using \<open>s2 \<in> io_targets M2 (initial M2) (vs @ xs2)\<close> by auto | |
have "productF M2 M1 FAIL PM" | |
using assms(4) by auto | |
have "well_formed M1" | |
using assms(2) by auto | |
have "well_formed M2" | |
using assms(3) by auto | |
have "observable PM" | |
by (meson assms(2) assms(3) assms(4) observable_productF) | |
have "length (vs@xs1) = length tr2_1" | |
using \<open>length tr2_1 = length (vs @ xs1)\<close> by presburger | |
then have "length tr2_1 = length tr1_1" | |
using \<open>length tr1_1 = length (vs@xs1)\<close> by presburger | |
have "vs@xs1 \<in> L PM" | |
using productF_path_inclusion[OF \<open>length (vs@xs1) = length tr2_1\<close> \<open>length tr2_1 = length tr1_1\<close> | |
\<open>productF M2 M1 FAIL PM\<close> \<open>well_formed M2\<close> \<open>well_formed M1\<close>] | |
by (meson Int_iff \<open>productF M2 M1 FAIL PM\<close> \<open>vs @ xs1 \<in> L M1\<close> \<open>vs @ xs1 \<in> L M2\<close> \<open>well_formed M1\<close> | |
\<open>well_formed M2\<close> productF_language) | |
have "length (vs@xs2) = length tr2_2" | |
using \<open>length tr2_2 = length (vs @ xs2)\<close> by presburger | |
then have "length tr2_2 = length tr1_2" | |
using \<open>length tr1_2 = length (vs@xs2)\<close> by presburger | |
have "vs@xs2 \<in> L PM" | |
using productF_path_inclusion[OF \<open>length (vs@xs2) = length tr2_2\<close> \<open>length tr2_2 = length tr1_2\<close> | |
\<open>productF M2 M1 FAIL PM\<close> \<open>well_formed M2\<close> \<open>well_formed M1\<close>] | |
by (meson Int_iff \<open>productF M2 M1 FAIL PM\<close> \<open>vs @ xs2 \<in> L M1\<close> \<open>vs @ xs2 \<in> L M2\<close> \<open>well_formed M1\<close> | |
\<open>well_formed M2\<close> productF_language) | |
have "io_targets PM (initial M2, initial M1) (vs @ xs1) = {(s2, s1)}" | |
using productF_path_io_targets_reverse | |
[OF \<open>productF M2 M1 FAIL PM\<close> \<open>s2 \<in> io_targets M2 (initial M2) (vs @ xs1)\<close> | |
\<open>s1 \<in> io_targets M1 (initial M1) (vs @ xs1)\<close> \<open>vs @ xs1 \<in> L M2\<close> \<open>vs @ xs1 \<in> L M1\<close> ] | |
proof - | |
have "\<forall>c f. c \<noteq> initial (f::('a, 'b, 'c) FSM) \<or> c \<in> nodes f" | |
by blast | |
then show ?thesis | |
by (metis (no_types) \<open>\<lbrakk>observable M2; observable M1; well_formed M2; well_formed M1; | |
initial M2 \<in> nodes M2; initial M1 \<in> nodes M1\<rbrakk> | |
\<Longrightarrow> io_targets PM (initial M2, initial M1) (vs @ xs1) = {(s2, s1)}\<close> | |
assms(2) assms(3)) | |
qed | |
have "io_targets PM (initial M2, initial M1) (vs @ xs2) = {(s2, s1)}" | |
using productF_path_io_targets_reverse | |
[OF \<open>productF M2 M1 FAIL PM\<close> \<open>s2 \<in> io_targets M2 (initial M2) (vs @ xs2)\<close> | |
\<open>s1 \<in> io_targets M1 (initial M1) (vs @ xs2)\<close> \<open>vs @ xs2 \<in> L M2\<close> \<open>vs @ xs2 \<in> L M1\<close> ] | |
proof - | |
have "\<forall>c f. c \<noteq> initial (f::('a, 'b, 'c) FSM) \<or> c \<in> nodes f" | |
by blast | |
then show ?thesis | |
by (metis (no_types) \<open>\<lbrakk>observable M2; observable M1; well_formed M2; well_formed M1; | |
initial M2 \<in> nodes M2; initial M1 \<in> nodes M1\<rbrakk> | |
\<Longrightarrow> io_targets PM (initial M2, initial M1) (vs @ xs2) = {(s2, s1)}\<close> | |
assms(2) assms(3)) | |
qed | |
have "prefix (vs @ xs1) (vs @ xs2)" | |
using \<open>prefix xs1 xs2\<close> by auto | |
have "sequence_to_failure M1 M2 (vs@xs)" | |
using assms(1) by auto | |
have "prefix (vs@xs1) (vs@xs')" | |
using \<open>prefix xs1 xs2\<close> \<open>prefix xs2 xs'\<close> prefix_order.dual_order.trans same_prefix_prefix | |
by blast | |
have "prefix (vs@xs2) (vs@xs')" | |
using \<open>prefix xs2 xs'\<close> prefix_order.dual_order.trans same_prefix_prefix by blast | |
have "io_targets PM (initial PM) (vs @ xs1) = {(s2,s1)}" | |
using \<open>io_targets PM (initial M2, initial M1) (vs @ xs1) = {(s2, s1)}\<close> assms(4) by auto | |
have "io_targets PM (initial PM) (vs @ xs2) = {(s2,s1)}" | |
using \<open>io_targets PM (initial M2, initial M1) (vs @ xs2) = {(s2, s1)}\<close> assms(4) by auto | |
have "(vs @ xs2) @ (drop (length xs2) xs) = vs@xs" | |
by (metis \<open>prefix xs2 xs'\<close> append_eq_appendI append_eq_conv_conj assms(6) prefixE) | |
moreover have "io_targets PM (initial PM) (vs@xs) = {FAIL}" | |
using sequence_to_failure_reaches_FAIL_ob[OF \<open>sequence_to_failure M1 M2 (vs@xs)\<close> assms(2,3) | |
\<open>productF M2 M1 FAIL PM\<close>] | |
by assumption | |
ultimately have "io_targets PM (initial PM) ((vs @ xs2) @ (drop (length xs2) xs)) = {FAIL}" | |
by auto | |
have "io_targets PM (s2,s1) (drop (length xs2) xs) = {FAIL}" | |
using observable_io_targets_split | |
[OF \<open>observable PM\<close> | |
\<open>io_targets PM (initial PM) ((vs @ xs2) @ (drop (length xs2) xs)) = {FAIL}\<close> | |
\<open>io_targets PM (initial PM) (vs @ xs2) = {(s2, s1)}\<close>] | |
by assumption | |
have "io_targets PM (initial PM) (vs@xs1@(drop (length xs2) xs)) = {FAIL}" | |
using observable_io_targets_append | |
[OF \<open>observable PM\<close> \<open>io_targets PM (initial PM) (vs @ xs1) = {(s2,s1)}\<close> | |
\<open>io_targets PM (s2,s1) (drop (length xs2) xs) = {FAIL}\<close>] | |
by simp | |
have "sequence_to_failure M1 M2 (vs@xs1@(drop (length xs2) xs))" | |
using sequence_to_failure_alt_def | |
[OF \<open>io_targets PM (initial PM) (vs@xs1@(drop (length xs2) xs)) = {FAIL}\<close> assms(2,3)] | |
assms(4) | |
by blast | |
have "length xs1 < length xs2" | |
using \<open>prefix xs1 xs2\<close> \<open>xs1 \<noteq> xs2\<close> prefix_length_prefix by fastforce | |
have prefix_drop: "ys = ys1 @ (drop (length ys1)) ys" if "prefix ys1 ys" | |
for ys ys1 :: "('a \<times> 'b) list" | |
using that by (induction ys1) (auto elim: prefixE) | |
then have "xs = (xs1 @ (drop (length xs1) xs))" | |
using \<open>prefix xs1 xs2\<close> \<open>prefix xs2 xs'\<close> \<open>prefix xs' xs\<close> by simp | |
then have "length xs1 < length xs" | |
using prefix_drop[OF \<open>prefix xs2 xs'\<close>] \<open>prefix xs2 xs'\<close> \<open>prefix xs' xs\<close> | |
using \<open>length xs1 < length xs2\<close> | |
by (auto dest!: prefix_length_le) | |
have "length (xs1@(drop (length xs2) xs)) < length xs" | |
using \<open>length xs1 < length xs2\<close> \<open>length xs1 < length xs\<close> by auto | |
have "vs \<in> L\<^sub>i\<^sub>n M1 V | |
\<and> sequence_to_failure M1 M2 (vs @ xs1@(drop (length xs2) xs)) | |
\<and> length (xs1@(drop (length xs2) xs)) < length xs" | |
using \<open>length (xs1 @ drop (length xs2) xs) < length xs\<close> | |
\<open>sequence_to_failure M1 M2 (vs @ xs1 @ drop (length xs2) xs)\<close> | |
assms(1) minimal_sequence_to_failure_extending.simps | |
by blast | |
then have "\<not> minimal_sequence_to_failure_extending V M1 M2 vs xs" | |
by (meson minimal_sequence_to_failure_extending.elims(2)) | |
then show "False" | |
using assms(1) by linarith | |
qed | |
lemma minimal_sequence_to_failure_extending_implies_Rep_Cov : | |
assumes "minimal_sequence_to_failure_extending V M1 M2 vs xs" | |
and "OFSM M1" | |
and "OFSM M2" | |
and "test_tools M2 M1 FAIL PM V \<Omega>" | |
and "V'' \<in> N (vs@xsR) M1 V" | |
and "prefix xsR xs" | |
shows "\<not> Rep_Cov M2 M1 V'' vs xsR" | |
proof | |
assume "Rep_Cov M2 M1 V'' vs xsR" | |
then obtain xs' vs' s2 s1 where "xs' \<noteq> []" | |
"prefix xs' xsR" | |
"vs' \<in> V''" | |
"io_targets M2 (initial M2) (vs @ xs') = {s2}" | |
"io_targets M2 (initial M2) (vs') = {s2}" | |
"io_targets M1 (initial M1) (vs @ xs') = {s1}" | |
"io_targets M1 (initial M1) (vs') = {s1}" | |
by auto | |
then have "s2 \<in> io_targets M2 (initial M2) (vs @ xs')" | |
"s2 \<in> io_targets M2 (initial M2) (vs')" | |
"s1 \<in> io_targets M1 (initial M1) (vs @ xs')" | |
"s1 \<in> io_targets M1 (initial M1) (vs')" | |
by auto | |
have "vs@xs' \<in> L M1" | |
using io_target_implies_L[OF \<open>s1 \<in> io_targets M1 (initial M1) (vs @ xs')\<close>] by assumption | |
have "vs' \<in> L M1" | |
using io_target_implies_L[OF \<open>s1 \<in> io_targets M1 (initial M1) (vs')\<close>] by assumption | |
have "vs@xs' \<in> L M2" | |
using io_target_implies_L[OF \<open>s2 \<in> io_targets M2 (initial M2) (vs @ xs')\<close>] by assumption | |
have "vs' \<in> L M2" | |
using io_target_implies_L[OF \<open>s2 \<in> io_targets M2 (initial M2) (vs')\<close>] by assumption | |
obtain tr1_1 where "path M1 (vs@xs' || tr1_1) (initial M1)" | |
"length tr1_1 = length (vs@xs')" | |
"target (vs@xs' || tr1_1) (initial M1) = s1" | |
using \<open>s1 \<in> io_targets M1 (initial M1) (vs @ xs')\<close> by auto | |
obtain tr1_2 where "path M1 (vs' || tr1_2) (initial M1)" | |
"length tr1_2 = length (vs')" | |
"target (vs' || tr1_2) (initial M1) = s1" | |
using \<open>s1 \<in> io_targets M1 (initial M1) (vs')\<close> by auto | |
obtain tr2_1 where "path M2 (vs@xs' || tr2_1) (initial M2)" | |
"length tr2_1 = length (vs@xs')" | |
"target (vs@xs' || tr2_1) (initial M2) = s2" | |
using \<open>s2 \<in> io_targets M2 (initial M2) (vs @ xs')\<close> by auto | |
obtain tr2_2 where "path M2 (vs' || tr2_2) (initial M2)" | |
"length tr2_2 = length (vs')" | |
"target (vs' || tr2_2) (initial M2) = s2" | |
using \<open>s2 \<in> io_targets M2 (initial M2) (vs')\<close> by auto | |
have "productF M2 M1 FAIL PM" | |
using assms(4) by auto | |
have "well_formed M1" | |
using assms(2) by auto | |
have "well_formed M2" | |
using assms(3) by auto | |
have "observable PM" | |
by (meson assms(2) assms(3) assms(4) observable_productF) | |
have "length (vs@xs') = length tr2_1" | |
using \<open>length tr2_1 = length (vs @ xs')\<close> by presburger | |
then have "length tr2_1 = length tr1_1" | |
using \<open>length tr1_1 = length (vs@xs')\<close> by presburger | |
have "vs@xs' \<in> L PM" | |
using productF_path_inclusion[OF \<open>length (vs@xs') = length tr2_1\<close> \<open>length tr2_1 = length tr1_1\<close> | |
\<open>productF M2 M1 FAIL PM\<close> \<open>well_formed M2\<close> \<open>well_formed M1\<close>] | |
by (meson Int_iff \<open>productF M2 M1 FAIL PM\<close> \<open>vs @ xs' \<in> L M1\<close> \<open>vs @ xs' \<in> L M2\<close> \<open>well_formed M1\<close> | |
\<open>well_formed M2\<close> productF_language) | |
have "length (vs') = length tr2_2" | |
using \<open>length tr2_2 = length (vs')\<close> by presburger | |
then have "length tr2_2 = length tr1_2" | |
using \<open>length tr1_2 = length (vs')\<close> by presburger | |
have "vs' \<in> L PM" | |
using productF_path_inclusion[OF \<open>length (vs') = length tr2_2\<close> \<open>length tr2_2 = length tr1_2\<close> | |
\<open>productF M2 M1 FAIL PM\<close> \<open>well_formed M2\<close> \<open>well_formed M1\<close>] | |
by (meson Int_iff \<open>productF M2 M1 FAIL PM\<close> \<open>vs' \<in> L M1\<close> \<open>vs' \<in> L M2\<close> \<open>well_formed M1\<close> | |
\<open>well_formed M2\<close> productF_language) | |
have "io_targets PM (initial M2, initial M1) (vs @ xs') = {(s2, s1)}" | |
using productF_path_io_targets_reverse | |
[OF \<open>productF M2 M1 FAIL PM\<close> \<open>s2 \<in> io_targets M2 (initial M2) (vs @ xs')\<close> | |
\<open>s1 \<in> io_targets M1 (initial M1) (vs @ xs')\<close> \<open>vs @ xs' \<in> L M2\<close> \<open>vs @ xs' \<in> L M1\<close> ] | |
proof - | |
have "\<forall>c f. c \<noteq> initial (f::('a, 'b, 'c) FSM) \<or> c \<in> nodes f" | |
by blast | |
then show ?thesis | |
by (metis (no_types) \<open>\<lbrakk>observable M2; observable M1; well_formed M2; well_formed M1; | |
initial M2 \<in> nodes M2; initial M1 \<in> nodes M1\<rbrakk> | |
\<Longrightarrow> io_targets PM (initial M2, initial M1) (vs @ xs') = {(s2, s1)}\<close> | |
assms(2) assms(3)) | |
qed | |
have "io_targets PM (initial M2, initial M1) (vs') = {(s2, s1)}" | |
using productF_path_io_targets_reverse | |
[OF \<open>productF M2 M1 FAIL PM\<close> \<open>s2 \<in> io_targets M2 (initial M2) (vs')\<close> | |
\<open>s1 \<in> io_targets M1 (initial M1) (vs')\<close> \<open>vs' \<in> L M2\<close> \<open>vs' \<in> L M1\<close> ] | |
proof - | |
have "\<forall>c f. c \<noteq> initial (f::('a, 'b, 'c) FSM) \<or> c \<in> nodes f" | |
by blast | |
then show ?thesis | |
by (metis (no_types) \<open>\<lbrakk>observable M2; observable M1; well_formed M2; well_formed M1; | |
initial M2 \<in> nodes M2; initial M1 \<in> nodes M1\<rbrakk> | |
\<Longrightarrow> io_targets PM (initial M2, initial M1) (vs') = {(s2, s1)}\<close> | |
assms(2) assms(3)) | |
qed | |
have "io_targets PM (initial PM) (vs') = {(s2, s1)}" | |
by (metis (no_types) \<open>io_targets PM (initial M2, initial M1) vs' = {(s2, s1)}\<close> | |
\<open>productF M2 M1 FAIL PM\<close> productF_simps(4)) | |
have "sequence_to_failure M1 M2 (vs@xs)" | |
using assms(1) by auto | |
have "xs = xs' @ (drop (length xs') xs)" | |
by (metis \<open>prefix xs' xsR\<close> append_assoc append_eq_conv_conj assms(6) prefixE) | |
then have "io_targets PM (initial M2, initial M1) (vs @ xs' @ (drop (length xs') xs)) = {FAIL}" | |
by (metis \<open>productF M2 M1 FAIL PM\<close> \<open>sequence_to_failure M1 M2 (vs @ xs)\<close> assms(2) assms(3) | |
productF_simps(4) sequence_to_failure_reaches_FAIL_ob) | |
then have "io_targets PM (initial M2, initial M1) ((vs @ xs') @ (drop (length xs') xs)) = {FAIL}" | |
by auto | |
have "io_targets PM (s2, s1) (drop (length xs') xs) = {FAIL}" | |
using observable_io_targets_split | |
[OF \<open>observable PM\<close> | |
\<open>io_targets PM (initial M2,initial M1) ((vs @ xs') @ (drop (length xs') xs)) = {FAIL}\<close> | |
\<open>io_targets PM (initial M2, initial M1) (vs @ xs') = {(s2, s1)}\<close>] | |
by assumption | |
have "io_targets PM (initial PM) (vs' @ (drop (length xs') xs)) = {FAIL}" | |
using observable_io_targets_append | |
[OF \<open>observable PM\<close> \<open>io_targets PM (initial PM) (vs') = {(s2, s1)}\<close> | |
\<open>io_targets PM (s2, s1) (drop (length xs') xs) = {FAIL}\<close>] | |
by assumption | |
have "sequence_to_failure M1 M2 (vs' @ (drop (length xs') xs))" | |
using sequence_to_failure_alt_def | |
[OF \<open>io_targets PM (initial PM) (vs' @ (drop (length xs') xs)) = {FAIL}\<close> assms(2,3)] | |
assms(4) | |
by blast | |
have "length (drop (length xs') xs) < length xs" | |
by (metis (no_types) \<open>xs = xs' @ drop (length xs') xs\<close> \<open>xs' \<noteq> []\<close> length_append | |
length_greater_0_conv less_add_same_cancel2) | |
have "vs' \<in> L\<^sub>i\<^sub>n M1 V" | |
proof - | |
have "V'' \<in> Perm V M1" | |
using assms(5) unfolding N.simps by blast | |
then obtain f where f_def : "V'' = image f V | |
\<and> (\<forall> v \<in> V . f v \<in> language_state_for_input M1 (initial M1) v)" | |
unfolding Perm.simps by blast | |
then obtain v where "v \<in> V" "vs' = f v" | |
using \<open>vs' \<in> V''\<close> by auto | |
then have "vs' \<in> language_state_for_input M1 (initial M1) v" | |
using f_def by auto | |
have "language_state_for_input M1 (initial M1) v = L\<^sub>i\<^sub>n M1 {v}" | |
by auto | |
moreover have "{v} \<subseteq> V" | |
using \<open>v \<in> V\<close> by blast | |
ultimately have "language_state_for_input M1 (initial M1) v \<subseteq> L\<^sub>i\<^sub>n M1 V" | |
unfolding language_state_for_inputs.simps language_state_for_input.simps by blast | |
then show ?thesis | |
using\<open>vs' \<in> language_state_for_input M1 (initial M1) v\<close> by blast | |
qed | |
have "\<not> minimal_sequence_to_failure_extending V M1 M2 vs xs" | |
using \<open>vs' \<in> L\<^sub>i\<^sub>n M1 V\<close> | |
\<open>sequence_to_failure M1 M2 (vs' @ (drop (length xs') xs))\<close> | |
\<open>length (drop (length xs') xs) < length xs\<close> | |
using minimal_sequence_to_failure_extending.elims(2) by blast | |
then show "False" | |
using assms(1) by linarith | |
qed | |
lemma mstfe_no_repetition : | |
assumes "minimal_sequence_to_failure_extending V M1 M2 vs xs" | |
and "OFSM M1" | |
and "OFSM M2" | |
and "test_tools M2 M1 FAIL PM V \<Omega>" | |
and "V'' \<in> N (vs@xs') M1 V" | |
and "prefix xs' xs" | |
shows "\<not> Rep_Pre M2 M1 vs xs'" | |
and "\<not> Rep_Cov M2 M1 V'' vs xs'" | |
using minimal_sequence_to_failure_extending_implies_Rep_Pre[OF assms] | |
minimal_sequence_to_failure_extending_implies_Rep_Cov[OF assms] | |
by linarith+ | |
subsection \<open> Sufficiency of the test suite to test for reduction \<close> | |
text \<open> | |
The following lemma proves that set of input sequences generated in the final iteration of the | |
@{verbatim TS} function constitutes a test suite sufficient to test for reduction the FSMs it has | |
been generated for. | |
This proof is performed by contradiction: If the test suite is not sufficient, then some minimal | |
sequence to a failure extending the deterministic state cover must exist. Due to the test suite | |
being assumed insufficient, this sequence cannot be contained in it and hence a prefix of it must | |
have been contained in one of the sets calculated by the @{verbatim R} function. This is only | |
possible if the prefix is not a minimal sequence to a failure extending the deterministic state | |
cover or if the test suite observes a failure, both of which violates the assumptions. | |
\<close> | |
lemma asc_sufficiency : | |
assumes "OFSM M1" | |
and "OFSM M2" | |
and "asc_fault_domain M2 M1 m" | |
and "test_tools M2 M1 FAIL PM V \<Omega>" | |
and "final_iteration M2 M1 \<Omega> V m i" | |
shows "M1 \<preceq>\<lbrakk>(TS M2 M1 \<Omega> V m i) . \<Omega>\<rbrakk> M2 \<longrightarrow> M1 \<preceq> M2" | |
proof | |
assume "atc_io_reduction_on_sets M1 (TS M2 M1 \<Omega> V m i) \<Omega> M2" | |
show "M1 \<preceq> M2" | |
proof (rule ccontr) | |
let ?TS = "\<lambda> n . TS M2 M1 \<Omega> V m n" | |
let ?C = "\<lambda> n . C M2 M1 \<Omega> V m n" | |
let ?RM = "\<lambda> n . RM M2 M1 \<Omega> V m n" | |
assume "\<not> M1 \<preceq> M2" | |
obtain vs xs where "minimal_sequence_to_failure_extending V M1 M2 vs xs" | |
using assms(1) assms(2) assms(4) | |
minimal_sequence_to_failure_extending_det_state_cover_ob[OF _ _ _ _ \<open>\<not> M1 \<preceq> M2\<close>, of V] | |
by blast | |
then have "vs \<in> L\<^sub>i\<^sub>n M1 V" | |
"sequence_to_failure M1 M2 (vs @ xs)" | |
"\<not> (\<exists> io' . \<exists> w' \<in> L\<^sub>i\<^sub>n M1 V . sequence_to_failure M1 M2 (w' @ io') | |
\<and> length io' < length xs)" | |
by auto | |
then have "vs@xs \<in> L M1 - L M2" | |
by auto | |
have "vs@xs \<in> L\<^sub>i\<^sub>n M1 {map fst (vs@xs)}" | |
by (metis (full_types) Diff_iff \<open>vs @ xs \<in> L M1 - L M2\<close> insertI1 | |
language_state_for_inputs_map_fst) | |
have "vs@xs \<notin> L\<^sub>i\<^sub>n M2 {map fst (vs@xs)}" | |
by (meson Diff_iff \<open>vs @ xs \<in> L M1 - L M2\<close> language_state_for_inputs_in_language_state | |
subsetCE) | |
have "finite V" | |
using det_state_cover_finite assms(4,2) by auto | |
then have "finite (?TS i)" | |
using TS_finite[of V M2] assms(2) by auto | |
then have "io_reduction_on M1 (?TS i) M2" | |
using io_reduction_from_atc_io_reduction | |
[OF \<open>atc_io_reduction_on_sets M1 (TS M2 M1 \<Omega> V m i) \<Omega> M2\<close>] | |
by auto | |
have "map fst (vs@xs) \<notin> ?TS i" | |
proof - | |
have f1: "\<forall>ps P Pa. (ps::('a \<times> 'b) list) \<notin> P - Pa \<or> ps \<in> P \<and> ps \<notin> Pa" | |
by blast | |
have "\<forall>P Pa ps. \<not> P \<subseteq> Pa \<or> (ps::('a \<times> 'b) list) \<in> Pa \<or> ps \<notin> P" | |
by blast | |
then show ?thesis | |
using f1 by (metis (no_types) \<open>vs @ xs \<in> L M1 - L M2\<close> \<open>io_reduction_on M1 (?TS i) M2\<close> | |
language_state_for_inputs_in_language_state language_state_for_inputs_map_fst) | |
qed | |
have "map fst vs \<in> V" | |
using \<open>vs \<in> L\<^sub>i\<^sub>n M1 V\<close> by auto | |
let ?stf = "map fst (vs@xs)" | |
let ?stfV = "map fst vs" | |
let ?stfX = "map fst xs" | |
have "?stf = ?stfV @ ?stfX" | |
by simp | |
then have "?stfV @ ?stfX \<notin> ?TS i" | |
using \<open>?stf \<notin> ?TS i\<close> by auto | |
have "mcp (?stfV @ ?stfX) V ?stfV" | |
by (metis \<open>map fst (vs @ xs) = map fst vs @ map fst xs\<close> | |
\<open>minimal_sequence_to_failure_extending V M1 M2 vs xs\<close> assms(1) assms(2) assms(4) | |
minimal_sequence_to_failure_extending_mcp) | |
have "set ?stf \<subseteq> inputs M1" | |
by (meson DiffD1 \<open>vs @ xs \<in> L M1 - L M2\<close> assms(1) language_state_inputs) | |
then have "set ?stf \<subseteq> inputs M2" | |
using assms(3) by blast | |
moreover have "set ?stf = set ?stfV \<union> set ?stfX" | |
by simp | |
ultimately have "set ?stfX \<subseteq> inputs M2" | |
by blast | |
obtain xr j where "xr \<noteq> ?stfX" | |
"prefix xr ?stfX" | |
"Suc j \<le> i" | |
"?stfV@xr \<in> RM M2 M1 \<Omega> V m (Suc j)" | |
using TS_non_containment_causes_final_suc[OF \<open>?stfV @ ?stfX \<notin> ?TS i\<close> | |
\<open>mcp (?stfV @ ?stfX) V ?stfV\<close> \<open>set ?stfX \<subseteq> inputs M2\<close> assms(5,2)] | |
by blast | |
let ?yr = "take (length xr) (map snd xs)" | |
have "length ?yr = length xr" | |
using \<open>prefix xr (map fst xs)\<close> prefix_length_le by fastforce | |
have "(xr || ?yr) = take (length xr) xs" | |
by (metis (no_types, opaque_lifting) \<open>prefix xr (map fst xs)\<close> append_eq_conv_conj prefixE take_zip | |
zip_map_fst_snd) | |
have "prefix (vs@(xr || ?yr)) (vs@xs)" | |
by (simp add: \<open>xr || take (length xr) (map snd xs) = take (length xr) xs\<close> take_is_prefix) | |
have "xr = take (length xr) (map fst xs)" | |
by (metis \<open>length (take (length xr) (map snd xs)) = length xr\<close> | |
\<open>xr || take (length xr) (map snd xs) = take (length xr) xs\<close> map_fst_zip take_map) | |
have "vs@(xr || ?yr) \<in> L M1" | |
by (metis DiffD1 \<open>prefix (vs @ (xr || take (length xr) (map snd xs))) (vs @ xs)\<close> | |
\<open>vs @ xs \<in> L M1 - L M2\<close> language_state_prefix prefixE) | |
then have "vs@(xr || ?yr) \<in> L\<^sub>i\<^sub>n M1 {?stfV @ xr}" | |
by (metis \<open>length (take (length xr) (map snd xs)) = length xr\<close> insertI1 | |
language_state_for_inputs_map_fst map_append map_fst_zip) | |
have "length xr < length xs" | |
by (metis \<open>xr = take (length xr) (map fst xs)\<close> \<open>xr \<noteq> map fst xs\<close> not_le_imp_less take_all | |
take_map) | |
from \<open>?stfV@xr \<in> RM M2 M1 \<Omega> V m (Suc j)\<close> have "?stfV@xr \<in> {xs' \<in> C M2 M1 \<Omega> V m (Suc j) . | |
(\<not> (L\<^sub>i\<^sub>n M1 {xs'} \<subseteq> L\<^sub>i\<^sub>n M2 {xs'})) | |
\<or> (\<forall> io \<in> L\<^sub>i\<^sub>n M1 {xs'} . | |
(\<exists> V'' \<in> N io M1 V . | |
(\<exists> S1 . | |
(\<exists> vs xs . | |
io = (vs@xs) | |
\<and> mcp (vs@xs) V'' vs | |
\<and> S1 \<subseteq> nodes M2 | |
\<and> (\<forall> s1 \<in> S1 . \<forall> s2 \<in> S1 . | |
s1 \<noteq> s2 \<longrightarrow> | |
(\<forall> io1 \<in> RP M2 s1 vs xs V'' . | |
\<forall> io2 \<in> RP M2 s2 vs xs V'' . | |
B M1 io1 \<Omega> \<noteq> B M1 io2 \<Omega> )) | |
\<and> m < LB M2 M1 vs xs (TS M2 M1 \<Omega> V m j \<union> V) S1 \<Omega> V'' ))))}" | |
unfolding RM.simps by blast | |
moreover have "\<forall> xs' \<in> ?C (Suc j) . L\<^sub>i\<^sub>n M1 {xs'} \<subseteq> L\<^sub>i\<^sub>n M2 {xs'}" | |
proof | |
fix xs' assume "xs' \<in> ?C (Suc j)" | |
from \<open>Suc j \<le> i\<close> have "?C (Suc j) \<subseteq> ?TS i" | |
using C_subset TS_subset by blast | |
then have "{xs'} \<subseteq> ?TS i" | |
using \<open>xs' \<in> ?C (Suc j)\<close> by blast | |
show "L\<^sub>i\<^sub>n M1 {xs'} \<subseteq> L\<^sub>i\<^sub>n M2 {xs'}" | |
using io_reduction_on_subset[OF \<open>io_reduction_on M1 (?TS i) M2\<close> \<open>{xs'} \<subseteq> ?TS i\<close>] | |
by assumption | |
qed | |
ultimately have "(\<forall> io \<in> L\<^sub>i\<^sub>n M1 {?stfV@xr} . | |
(\<exists> V'' \<in> N io M1 V . | |
(\<exists> S1 . | |
(\<exists> vs xs . | |
io = (vs@xs) | |
\<and> mcp (vs@xs) V'' vs | |
\<and> S1 \<subseteq> nodes M2 | |
\<and> (\<forall> s1 \<in> S1 . \<forall> s2 \<in> S1 . | |
s1 \<noteq> s2 \<longrightarrow> | |
(\<forall> io1 \<in> RP M2 s1 vs xs V'' . | |
\<forall> io2 \<in> RP M2 s2 vs xs V'' . | |
B M1 io1 \<Omega> \<noteq> B M1 io2 \<Omega> )) | |
\<and> m < LB M2 M1 vs xs (TS M2 M1 \<Omega> V m j \<union> V) S1 \<Omega> V'' ))))" | |
by blast | |
then have " | |
(\<exists> V'' \<in> N (vs@(xr || ?yr)) M1 V . | |
(\<exists> S1 . | |
(\<exists> vs' xs' . | |
vs@(xr || ?yr) = (vs'@xs') | |
\<and> mcp (vs'@xs') V'' vs' | |
\<and> S1 \<subseteq> nodes M2 | |
\<and> (\<forall> s1 \<in> S1 . \<forall> s2 \<in> S1 . | |
s1 \<noteq> s2 \<longrightarrow> | |
(\<forall> io1 \<in> RP M2 s1 vs' xs' V'' . | |
\<forall> io2 \<in> RP M2 s2 vs' xs' V'' . | |
B M1 io1 \<Omega> \<noteq> B M1 io2 \<Omega> )) | |
\<and> m < LB M2 M1 vs' xs' (TS M2 M1 \<Omega> V m j \<union> V) S1 \<Omega> V'' )))" | |
using \<open>vs@(xr || ?yr) \<in> L\<^sub>i\<^sub>n M1 {?stfV @ xr}\<close> | |
by blast | |
then obtain V'' S1 vs' xs' where RM_impl : | |
"V'' \<in> N (vs@(xr || ?yr)) M1 V" | |
"vs@(xr || ?yr) = (vs'@xs')" | |
"mcp (vs'@xs') V'' vs'" | |
"S1 \<subseteq> nodes M2" | |
"(\<forall> s1 \<in> S1 . \<forall> s2 \<in> S1 . | |
s1 \<noteq> s2 \<longrightarrow> | |
(\<forall> io1 \<in> RP M2 s1 vs' xs' V'' . | |
\<forall> io2 \<in> RP M2 s2 vs' xs' V'' . | |
B M1 io1 \<Omega> \<noteq> B M1 io2 \<Omega> ))" | |
" m < LB M2 M1 vs' xs' (TS M2 M1 \<Omega> V m j \<union> V) S1 \<Omega> V''" | |
by blast | |
have "?stfV = mcp' (map fst (vs @ (xr || take (length xr) (map snd xs)))) V" | |
by (metis (full_types) \<open>length (take (length xr) (map snd xs)) = length xr\<close> | |
\<open>mcp (map fst vs @ map fst xs) V (map fst vs)\<close> \<open>prefix xr (map fst xs)\<close> map_append | |
map_fst_zip mcp'_intro mcp_prefix_of_suffix) | |
have "is_det_state_cover M2 V" | |
using assms(4) by blast | |
moreover have "well_formed M2" | |
using assms(2) by auto | |
moreover have "finite V" | |
using det_state_cover_finite assms(4,2) by auto | |
ultimately have "vs \<in> V''" | |
"vs = mcp' (vs @ (xr || take (length xr) (map snd xs))) V''" | |
using N_mcp_prefix[OF \<open>?stfV = mcp' (map fst (vs @ (xr || take (length xr) (map snd xs)))) V\<close> | |
\<open>V'' \<in> N (vs@(xr || ?yr)) M1 V\<close>, of M2] | |
by simp+ | |
have "vs' = vs" | |
by (metis (no_types) \<open>mcp (vs' @ xs') V'' vs'\<close> | |
\<open>vs = mcp' (vs @ (xr || take (length xr) (map snd xs))) V''\<close> | |
\<open>vs @ (xr || take (length xr) (map snd xs)) = vs' @ xs'\<close> mcp'_intro) | |
then have "xs' = (xr || ?yr)" | |
using \<open>vs @ (xr || take (length xr) (map snd xs)) = vs' @ xs'\<close> by blast | |
have "V \<subseteq> ?TS i" | |
proof - | |
have "1 \<le> i" | |
using \<open>Suc j \<le> i\<close> by linarith | |
then have "?TS 1 \<subseteq> ?TS i" | |
using TS_subset by blast | |
then show ?thesis | |
by auto | |
qed | |
have "?stfV@xr \<in> ?C (Suc j)" | |
using \<open>?stfV@xr \<in> RM M2 M1 \<Omega> V m (Suc j)\<close> unfolding RM.simps by blast | |
\<comment> \<open>show that the prerequisites (@{verbatim Prereq}) for @{verbatim LB} are met by construction\<close> | |
have "(\<forall>vs'a\<in>V''. prefix vs'a (vs' @ xs') \<longrightarrow> length vs'a \<le> length vs')" | |
using \<open>mcp (vs' @ xs') V'' vs'\<close> by auto | |
moreover have "atc_io_reduction_on_sets M1 (?TS j \<union> V) \<Omega> M2" | |
proof - | |
have "j < i" | |
using \<open>Suc j \<le> i\<close> by auto | |
then have "?TS j \<subseteq> ?TS i" | |
by (simp add: TS_subset) | |
then show ?thesis | |
using atc_io_reduction_on_subset | |
[OF \<open>atc_io_reduction_on_sets M1 (TS M2 M1 \<Omega> V m i) \<Omega> M2\<close>, of "?TS j"] | |
by (meson Un_subset_iff \<open>V \<subseteq> ?TS i\<close> \<open>atc_io_reduction_on_sets M1 (TS M2 M1 \<Omega> V m i) \<Omega> M2\<close> | |
atc_io_reduction_on_subset) | |
qed | |
moreover have "finite (?TS j \<union> V)" | |
proof - | |
have "finite (?TS j)" | |
using TS_finite[OF \<open>finite V\<close>, of M2 M1 \<Omega> m j] assms(2) by auto | |
then show ?thesis | |
using \<open>finite V\<close> by blast | |
qed | |
moreover have "V \<subseteq> ?TS j \<union> V" | |
by blast | |
moreover have "(\<forall> p . (prefix p xs' \<and> p \<noteq> xs') \<longrightarrow> map fst (vs' @ p) \<in> ?TS j \<union> V)" | |
proof | |
fix p | |
show "prefix p xs' \<and> p \<noteq> xs' \<longrightarrow> map fst (vs' @ p) \<in> TS M2 M1 \<Omega> V m j \<union> V" | |
proof | |
assume "prefix p xs' \<and> p \<noteq> xs'" | |
have "prefix (map fst (vs' @ p)) (map fst (vs' @ xs'))" | |
by (simp add: \<open>prefix p xs' \<and> p \<noteq> xs'\<close> map_mono_prefix) | |
have "prefix (map fst (vs' @ p)) (?stfV @ xr)" | |
using \<open>length (take (length xr) (map snd xs)) = length xr\<close> | |
\<open>prefix (map fst (vs' @ p)) (map fst (vs' @ xs'))\<close> | |
\<open>vs' = vs\<close> \<open>xs' = xr || take (length xr) (map snd xs)\<close> | |
by auto | |
then have "prefix (map fst vs' @ map fst p) (?stfV @ xr)" | |
by simp | |
then have "prefix (map fst p) xr" | |
by (simp add: \<open>vs' = vs\<close>) | |
have "?stfV @ xr \<in> ?TS (Suc j)" | |
proof (cases j) | |
case 0 | |
then show ?thesis | |
using \<open>map fst vs @ xr \<in> C M2 M1 \<Omega> V m (Suc j)\<close> by auto | |
next | |
case (Suc nat) | |
then show ?thesis | |
using TS.simps(3) \<open>map fst vs @ xr \<in> C M2 M1 \<Omega> V m (Suc j)\<close> by blast | |
qed | |
have "mcp (map fst vs @ xr) V (map fst vs)" | |
using \<open>mcp (map fst vs @ map fst xs) V (map fst vs)\<close> \<open>prefix xr (map fst xs)\<close> | |
mcp_prefix_of_suffix | |
by blast | |
have "map fst vs @ map fst p \<in> TS M2 M1 \<Omega> V m (Suc j)" | |
using TS_prefix_containment[OF \<open>?stfV @ xr \<in> ?TS (Suc j)\<close> | |
\<open>mcp (map fst vs @ xr) V (map fst vs)\<close> | |
\<open>prefix (map fst p) xr\<close>] | |
by assumption | |
have "Suc (length xr) = (Suc j)" | |
using C_index[OF \<open>?stfV@xr \<in> ?C (Suc j)\<close> \<open>mcp (map fst vs @ xr) V (map fst vs)\<close>] | |
by assumption | |
have"Suc (length p) < (Suc j)" | |
proof - | |
have "map fst xs' = xr" | |
by (metis \<open>xr = take (length xr) (map fst xs)\<close> | |
\<open>xr || take (length xr) (map snd xs) = take (length xr) xs\<close> | |
\<open>xs' = xr || take (length xr) (map snd xs)\<close> take_map) | |
then show ?thesis | |
by (metis (no_types) Suc_less_eq \<open>Suc (length xr) = Suc j\<close> \<open>prefix p xs' \<and> p \<noteq> xs'\<close> | |
append_eq_conv_conj length_map nat_less_le prefixE prefix_length_le take_all) | |
qed | |
have "mcp (map fst vs @ map fst p) V (map fst vs)" | |
using \<open>mcp (map fst vs @ xr) V (map fst vs)\<close> \<open>prefix (map fst p) xr\<close> mcp_prefix_of_suffix | |
by blast | |
then have "map fst vs @ map fst p \<in> ?C (Suc (length (map fst p)))" | |
using TS_index(2)[OF \<open>map fst vs @ map fst p \<in> TS M2 M1 \<Omega> V m (Suc j)\<close>] by auto | |
have "map fst vs @ map fst p \<in> ?TS j" | |
using TS_union[of M2 M1 \<Omega> V m j] | |
proof - | |
have "Suc (length p) \<in> {0..<Suc j}" | |
using \<open>Suc (length p) < Suc j\<close> by force | |
then show ?thesis | |
by (metis UN_I \<open>TS M2 M1 \<Omega> V m j = (\<Union>j\<in>set [0..<Suc j]. C M2 M1 \<Omega> V m j)\<close> | |
\<open>map fst vs @ map fst p \<in> C M2 M1 \<Omega> V m (Suc (length (map fst p)))\<close> | |
length_map set_upt) | |
qed | |
then show "map fst (vs' @ p) \<in> TS M2 M1 \<Omega> V m j \<union> V" | |
by (simp add: \<open>vs' = vs\<close>) | |
qed | |
qed | |
moreover have "vs' @ xs' \<in> L M2 \<inter> L M1" | |
by (metis (no_types, lifting) IntI RM_impl(2) | |
\<open>\<forall>xs'\<in>C M2 M1 \<Omega> V m (Suc j). L\<^sub>i\<^sub>n M1 {xs'} \<subseteq> L\<^sub>i\<^sub>n M2 {xs'}\<close> | |
\<open>map fst vs @ xr \<in> C M2 M1 \<Omega> V m (Suc j)\<close> | |
\<open>vs @ (xr || take (length xr) (map snd xs)) \<in> L\<^sub>i\<^sub>n M1 {map fst vs @ xr}\<close> | |
language_state_for_inputs_in_language_state subsetCE) | |
ultimately have "Prereq M2 M1 vs' xs' (?TS j \<union> V) S1 \<Omega> V''" | |
using RM_impl(4,5) unfolding Prereq.simps by blast | |
have "V'' \<in> Perm V M1" | |
using \<open>V'' \<in> N (vs@(xr || ?yr)) M1 V\<close> unfolding N.simps by blast | |
have \<open>prefix (xr || ?yr) xs\<close> | |
by (simp add: \<open>xr || take (length xr) (map snd xs) = take (length xr) xs\<close> take_is_prefix) | |
\<comment> \<open> show that furthermore neither @{verbatim Rep_Pre} nor @{verbatim Rep_Cov} holds \<close> | |
have "\<not> Rep_Pre M2 M1 vs (xr || ?yr)" | |
using minimal_sequence_to_failure_extending_implies_Rep_Pre | |
[OF \<open>minimal_sequence_to_failure_extending V M1 M2 vs xs\<close> assms(1,2) | |
\<open>test_tools M2 M1 FAIL PM V \<Omega>\<close> RM_impl(1) | |
\<open>prefix (xr || take (length xr) (map snd xs)) xs\<close>] | |
by assumption | |
then have "\<not> Rep_Pre M2 M1 vs' xs'" | |
using \<open>vs' = vs\<close> \<open>xs' = xr || ?yr\<close> by blast | |
have "\<not> Rep_Cov M2 M1 V'' vs (xr || ?yr)" | |
using minimal_sequence_to_failure_extending_implies_Rep_Cov | |
[OF \<open>minimal_sequence_to_failure_extending V M1 M2 vs xs\<close> assms(1,2) | |
\<open>test_tools M2 M1 FAIL PM V \<Omega>\<close> RM_impl(1) | |
\<open>prefix (xr || take (length xr) (map snd xs)) xs\<close>] | |
by assumption | |
then have "\<not> Rep_Cov M2 M1 V'' vs' xs'" | |
using \<open>vs' = vs\<close> \<open>xs' = xr || ?yr\<close> by blast | |
have "vs'@xs' \<in> L M1" | |
using \<open>vs @ (xr || take (length xr) (map snd xs)) \<in> L M1\<close> | |
\<open>vs' = vs\<close> \<open>xs' = xr || take (length xr) (map snd xs)\<close> | |
by blast | |
\<comment> \<open> therefore it is impossible to remove the prefix of the minimal sequence to a failure, | |
as this would require @{verbatim M1} to have more than m states \<close> | |
have "LB M2 M1 vs' xs' (?TS j \<union> V) S1 \<Omega> V'' \<le> card (nodes M1)" | |
using LB_count[OF \<open>vs'@xs' \<in> L M1\<close> assms(1,2,3) \<open>test_tools M2 M1 FAIL PM V \<Omega>\<close> | |
\<open>V'' \<in> Perm V M1\<close> \<open>Prereq M2 M1 vs' xs' (?TS j \<union> V) S1 \<Omega> V''\<close> | |
\<open>\<not> Rep_Pre M2 M1 vs' xs'\<close> \<open> \<not> Rep_Cov M2 M1 V'' vs' xs'\<close>] | |
by assumption | |
then have "LB M2 M1 vs' xs' (?TS j \<union> V) S1 \<Omega> V'' \<le> m" | |
using assms(3) by linarith | |
then show "False" | |
using \<open>m < LB M2 M1 vs' xs' (?TS j \<union> V) S1 \<Omega> V''\<close> by linarith | |
qed | |
qed | |
subsection \<open> Main result \<close> | |
text \<open> | |
The following lemmata add to the previous result to show that some FSM @{verbatim M1} is a reduction | |
of FSM @{verbatim M2} if and only if it is a reduction on the test suite generated by the adaptive | |
state counting algorithm for these FSMs. | |
\<close> | |
lemma asc_soundness : | |
assumes "OFSM M1" | |
and "OFSM M2" | |
shows "M1 \<preceq> M2 \<longrightarrow> atc_io_reduction_on_sets M1 T \<Omega> M2" | |
using atc_io_reduction_on_sets_reduction assms by blast | |
lemma asc_main_theorem : | |
assumes "OFSM M1" | |
and "OFSM M2" | |
and "asc_fault_domain M2 M1 m" | |
and "test_tools M2 M1 FAIL PM V \<Omega>" | |
and "final_iteration M2 M1 \<Omega> V m i" | |
shows "M1 \<preceq> M2 \<longleftrightarrow> atc_io_reduction_on_sets M1 (TS M2 M1 \<Omega> V m i) \<Omega> M2" | |
by (metis asc_sufficiency assms(1-5) atc_io_reduction_on_sets_reduction) | |
end |