--- a/IOA/example/Correctness.ML Tue Oct 24 14:59:17 1995 +0100
+++ /dev/null Thu Jan 01 00:00:00 1970 +0000
@@ -1,103 +0,0 @@
-(* Title: HOL/IOA/example/Correctness.ML
- ID: $Id$
- Author: Tobias Nipkow & Konrad Slind
- Copyright 1994 TU Muenchen
-
-The main correctness proof: Impl implements Spec
-*)
-
-open Impl;
-open Spec;
-
-val hom_ss = impl_ss;
-val hom_ioas = [Spec.ioa_def, Spec.trans_def,
- Sender.sender_trans_def,Receiver.receiver_trans_def]
- @ impl_ioas;
-
-val hom_ss' = hom_ss addsimps hom_ioas;
-
-val impl_asigs = [Sender.sender_asig_def,Receiver.receiver_asig_def,
- Channels.srch_asig_def,Channels.rsch_asig_def];
-
-(* A lemma about restricting the action signature of the implementation
- * to that of the specification.
- ****************************)
-goal Correctness.thy
- "a:externals(asig_of(restrict(impl_ioa,externals(spec_sig)))) = \
-\ (case a of \
-\ S_msg(m) => True \
-\ | R_msg(m) => True \
-\ | S_pkt(pkt) => False \
-\ | R_pkt(pkt) => False \
-\ | S_ack(b) => False \
-\ | R_ack(b) => False \
-\ | C_m_s => False \
-\ | C_m_r => False \
-\ | C_r_s => False \
-\ | C_r_r(m) => False)";
- by(simp_tac (hom_ss addcongs [if_weak_cong]
- addsimps ([externals_def, restrict_def, restrict_asig_def,
- asig_of_par, asig_comp_def, Spec.sig_def] @
- asig_projections @ impl_ioas @ impl_asigs)) 1);
- by(Action.action.induct_tac "a" 1);
- by(ALLGOALS(simp_tac (action_ss addsimps
- (actions_def :: asig_projections @ set_lemmas))));
-qed "externals_lemma";
-
-
-val sels = [Sender.sbit_def, Sender.sq_def, Sender.ssending_def,
- Receiver.rbit_def, Receiver.rq_def, Receiver.rsending_def];
-
-(* Proof of correctness *)
-goalw Correctness.thy [Spec.ioa_def, Solve.is_weak_pmap_def]
- "is_weak_pmap(hom, restrict(impl_ioa,externals(spec_sig)), spec_ioa)";
-by(simp_tac (hom_ss addsimps
- (Correctness.hom_def::[cancel_restrict,externals_lemma])) 1);
-br conjI 1;
-by(simp_tac (hom_ss addsimps impl_ioas) 1);
-br ballI 1;
-bd CollectD 1;
-by(asm_simp_tac (hom_ss addsimps sels) 1);
-by(REPEAT(rtac allI 1));
-br imp_conj_lemma 1; (* from lemmas.ML *)
-by(Action.action.induct_tac "a" 1);
-by(asm_simp_tac (hom_ss' setloop (split_tac [expand_if])) 1);
-by(forward_tac [inv4] 1);
-by(asm_full_simp_tac (hom_ss addsimps
- [imp_ex_equiv,neq_Nil_conv,ex_all_equiv]) 1);
-by(simp_tac hom_ss' 1);
-by(simp_tac hom_ss' 1);
-by(simp_tac hom_ss' 1);
-by(simp_tac hom_ss' 1);
-by(simp_tac hom_ss' 1);
-by(simp_tac hom_ss' 1);
-by(simp_tac hom_ss' 1);
-
-by(asm_simp_tac hom_ss' 1);
-by(forward_tac [inv4] 1);
-by(forward_tac [inv2] 1);
-be disjE 1;
-by(asm_simp_tac hom_ss 1);
-by(asm_full_simp_tac (hom_ss addsimps
- [imp_ex_equiv,neq_Nil_conv,ex_all_equiv]) 1);
-
-by(asm_simp_tac hom_ss' 1);
-by(forward_tac [inv2] 1);
-be disjE 1;
-
-by(forward_tac [inv3] 1);
-by(case_tac "sq(sen(s))=[]" 1);
-
-by(asm_full_simp_tac hom_ss' 1);
-by(fast_tac (HOL_cs addSDs [add_leD1 RS leD]) 1);
-
-by(case_tac "m = hd(sq(sen(s)))" 1);
-
-by(asm_full_simp_tac (hom_ss addsimps
- [imp_ex_equiv,neq_Nil_conv,ex_all_equiv]) 1);
-
-by(asm_full_simp_tac hom_ss 1);
-by(fast_tac (HOL_cs addSDs [add_leD1 RS leD]) 1);
-
-by(asm_full_simp_tac hom_ss 1);
-result();