X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=helm%2Fsoftware%2Fmatita%2Fcontribs%2Fng_assembly%2Femulator%2Fopcodes%2FRS08_table_tests.ma;h=73f1c0ad23372656977e38dd8e709fb2ef52ce42;hb=7f89b4dce54266c281479a14c01edc4bd33993d1;hp=155c6abf2a5168db766980831752830fc3d93342;hpb=a581a54f6118908a21ed3f960c70a0a2c863ca89;p=helm.git diff --git a/helm/software/matita/contribs/ng_assembly/emulator/opcodes/RS08_table_tests.ma b/helm/software/matita/contribs/ng_assembly/emulator/opcodes/RS08_table_tests.ma index 155c6abf2..73f1c0ad2 100755 --- a/helm/software/matita/contribs/ng_assembly/emulator/opcodes/RS08_table_tests.ma +++ b/helm/software/matita/contribs/ng_assembly/emulator/opcodes/RS08_table_tests.ma @@ -36,31 +36,35 @@ ndefinition RS08_not_impl_byte ≝ ]. (* test bytecode non implementati *) -nlemma ok_byte_table_RS08 : forall_b8 (λb. +(* !!! per brevita... *) +(*nlemma ok_byte_table_RS08 : forall_b8 (λb. (test_not_impl_byte b RS08_not_impl_byte ⊙ eq_w16 (get_byte_count RS08 b 〈〈x0,x0〉:〈x0,x0〉〉 opcode_table_RS08) 〈〈x0,x0〉:〈x0,x1〉〉) ⊗ (⊖ (test_not_impl_byte b RS08_not_impl_byte) ⊙ eq_w16 (get_byte_count RS08 b 〈〈x0,x0〉:〈x0,x0〉〉 opcode_table_RS08) 〈〈x0,x0〉:〈x0,x0〉〉)) = true. napply refl_eq. -nqed. +nqed.*) (* tutti op implementati *) -nlemma ok_pseudo_table_RS08 : +(* !!! per brevita... *) +(*nlemma ok_pseudo_table_RS08 : forall_op RS08 (λo. le_w16 〈〈x0,x0〉:〈x0,x1〉〉 (get_pseudo_count RS08 o 〈〈x0,x0〉:〈x0,x0〉〉 opcode_table_RS08)) = true. napply refl_eq. -nqed. +nqed.*) (* tutte im implementate *) -nlemma ok_mode_table_RS08 : +(* !!! per brevita... *) +(*nlemma ok_mode_table_RS08 : forall_im RS08 (λi. le_w16 〈〈x0,x0〉:〈x0,x1〉〉 (get_mode_count RS08 i 〈〈x0,x0〉:〈x0,x0〉〉 opcode_table_RS08)) = true. napply refl_eq. -nqed. +nqed.*) (* nessuna ripetizione di combinazione op + imm *) -nlemma ok_OpIm_table_RS08 : +(* !!! per brevita... *) +(*nlemma ok_OpIm_table_RS08 : forall_im RS08 (λi. forall_op RS08 (λo. le_w16 (get_OpIm_count RS08 o i 〈〈x0,x0〉:〈x0,x0〉〉 opcode_table_RS08) 〈〈x0,x0〉:〈x0,x1〉〉)) = true. napply refl_eq. -nqed. +nqed.*)