src/HOLCF/IOA/meta_theory/LiveIOA.ML
author paulson
Fri, 11 Dec 1998 10:38:51 +0100
changeset 6023 832b9269dedd
parent 5976 44290b71a85f
child 6161 bc2a76ce1ea3
permissions -rw-r--r--
deleted unclosed comment
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
4559
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     1
(*  Title:      HOLCF/IOA/meta_theory/LiveIOA.ML
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     2
    ID:         $Id$
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     3
    Author:     Olaf M"uller
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     4
    Copyright   1997  TU Muenchen
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     5
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     6
Live I/O Automata
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     7
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     8
*)   
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
     9
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    10
Delsimps [split_paired_Ex];
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    11
5068
fb28eaa07e01 isatool fixgoal;
wenzelm
parents: 4559
diff changeset
    12
Goalw [live_implements_def] 
4559
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    13
"!! A. [| live_implements (A,LA) (B,LB); live_implements (B,LB) (C,LC) |] \
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    14
\     ==> live_implements (A,LA) (C,LC)"; 
5132
24f992a25adc isatool expandshort;
wenzelm
parents: 5068
diff changeset
    15
by Auto_tac;
4559
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    16
qed"live_implements_trans";
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    17
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    18
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    19
section "Correctness of live refmap";
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    20
	
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    21
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    22
(* ---------------------------------------------------------------- *)
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    23
(*                Correctness of live refmap                        *)
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    24
(* ---------------------------------------------------------------- *)
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    25
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    26
5068
fb28eaa07e01 isatool fixgoal;
wenzelm
parents: 4559
diff changeset
    27
Goal "!! f. [| inp(C)=inp(A); out(C)=out(A); \
4559
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    28
\                  is_live_ref_map f (C,M) (A,L) |] \
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    29
\               ==> live_implements (C,M) (A,L)";
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    30
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    31
by (asm_full_simp_tac (simpset() addsimps [is_live_ref_map_def, live_implements_def,
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    32
livetraces_def,liveexecutions_def]) 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    33
by (safe_tac set_cs);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    34
by (res_inst_tac[("x","corresp_ex A f ex")] exI 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    35
by (safe_tac set_cs);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    36
  (* Traces coincide, Lemma 1 *)
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    37
  by (pair_tac "ex" 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    38
  by (etac (lemma_1 RS spec RS mp) 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    39
  by (simp_tac (simpset() addsimps [externals_def])1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    40
  by (SELECT_GOAL (auto_tac (claset(),simpset()))1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    41
  by (asm_full_simp_tac (simpset() addsimps [executions_def,reachable.reachable_0]) 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    42
 
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    43
  (* corresp_ex is execution, Lemma 2 *)
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    44
  by (pair_tac "ex" 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    45
  by (asm_full_simp_tac (simpset() addsimps [executions_def]) 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    46
  (* start state *) 
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    47
  by (rtac conjI 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    48
  by (asm_full_simp_tac (simpset() addsimps [is_ref_map_def,corresp_ex_def]) 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    49
  (* is-execution-fragment *)
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    50
  by (etac (lemma_2 RS spec RS mp) 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    51
  by (asm_full_simp_tac (simpset() addsimps [reachable.reachable_0]) 1);
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    52
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    53
 (* Liveness *)
5132
24f992a25adc isatool expandshort;
wenzelm
parents: 5068
diff changeset
    54
by Auto_tac;
4559
8e604d885b54 added files containing temproal logic and abstraction;
mueller
parents:
diff changeset
    55
qed"live_implements";