src/HOL/UNITY/Reach.ML
author wenzelm
Fri, 31 Jul 1998 11:03:31 +0200
changeset 5228 66925577cefe
parent 5196 1dd4ec921f71
child 5232 e5a7cdd07ea5
permissions -rw-r--r--
isatool expandshort;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     1
(*  Title:      HOL/UNITY/Reach.thy
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     2
    ID:         $Id$
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     4
    Copyright   1998  University of Cambridge
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     5
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     6
Reachability in Directed Graphs.  From Chandy and Misra, section 6.4.
4896
4727272f3db6 New syntax for function update; moved to main HOL directory
paulson
parents: 4776
diff changeset
     7
	[ this example took only four days!]
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     8
*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
     9
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    10
open Reach;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    11
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    12
(*TO SIMPDATA.ML??  FOR CLASET??  *)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    13
val major::prems = goal thy 
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    14
    "[| if P then Q else R;    \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    15
\       [| P;   Q |] ==> S;    \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    16
\       [| ~ P; R |] ==> S |] ==> S";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    17
by (cut_facts_tac [major] 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    18
by (blast_tac (claset() addSDs [if_bool_eq_disj RS iffD1] addIs prems) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    19
qed "ifE";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    20
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    21
AddSEs [ifE];
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    22
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    23
5196
1dd4ec921f71 update -> fun_upd
nipkow
parents: 5111
diff changeset
    24
val cmd_defs = [racts_def, asgt_def, fun_upd_def];
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    25
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
    26
Goalw [racts_def] "id : racts";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    27
by (Simp_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    28
qed "id_in_racts";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    29
AddIffs [id_in_racts];
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    30
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    31
(*All vertex sets are finite*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    32
AddIffs [[subset_UNIV, finite_graph] MRS finite_subset];
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    33
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    34
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    35
(** Constrains/Ensures tactics: NEED TO BE GENERALIZED OVER ALL PROGRAMS **)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    36
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    37
(*proves "constrains" properties when the program is specified*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    38
val constrains_tac = 
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    39
   SELECT_GOAL
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    40
      (EVERY [rtac constrainsI 1,
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    41
	      rewtac racts_def,
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    42
	      REPEAT_FIRST (eresolve_tac [insertE, emptyE]),
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    43
	      rewrite_goals_tac [racts_def, asgt_def],
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    44
	      ALLGOALS (SELECT_GOAL Auto_tac)]);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    45
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    46
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    47
(*proves "ensures" properties when the program is specified*)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    48
fun ensures_tac sact = 
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    49
    SELECT_GOAL
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    50
      (EVERY [REPEAT (resolve_tac [LeadsTo_Basis, leadsTo_Basis, ensuresI] 1),
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    51
	      res_inst_tac [("act", sact)] transient_mem 2,
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    52
	      Simp_tac 2,
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    53
	      constrains_tac 1,
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    54
	      rewrite_goals_tac [racts_def, asgt_def],
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    55
	      Auto_tac]);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    56
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    57
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
    58
Goalw [stable_def, invariant_def]
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    59
    "stable racts invariant";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    60
by (constrains_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    61
by (blast_tac (claset() addIs [r_into_rtrancl,rtrancl_trans]) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    62
qed "stable_invariant";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    63
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
    64
Goalw [rinit_def, invariant_def] "rinit <= invariant";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    65
by Auto_tac;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    66
qed "rinit_invariant";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    67
5111
8f4b72f0c15d Uncurried functions LeadsTo and reach
paulson
parents: 5071
diff changeset
    68
Goal "reachable (rinit,racts) <= invariant";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    69
by (simp_tac (simpset() addsimps
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    70
	      [strongest_invariant, stable_invariant, rinit_invariant]) 1); 
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    71
qed "reachable_subset_invariant";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    72
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    73
val reachable_subset_invariant' = 
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    74
    rewrite_rule [invariant_def] reachable_subset_invariant;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    75
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    76
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    77
(*** Fixedpoint ***)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    78
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    79
(*If it reaches a fixedpoint, it has found a solution*)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
    80
Goalw [fixedpoint_def, invariant_def]
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    81
    "fixedpoint Int invariant = { %v. (init, v) : edges^* }";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    82
by (rtac equalityI 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    83
by (blast_tac (claset() addIs [r_into_rtrancl,rtrancl_trans]) 2);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    84
by (auto_tac (claset() addSIs [ext], simpset()));
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    85
by (etac rtrancl_induct 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    86
by Auto_tac;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    87
qed "fixedpoint_invariant_correct";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    88
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
    89
Goalw (cmd_defs @ [FP_def, fixedpoint_def, stable_def, constrains_def])
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    90
    "FP racts <= fixedpoint";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    91
by Auto_tac;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    92
by (dtac bspec 1); 
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    93
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    94
by (asm_full_simp_tac (simpset() addsimps [Image_singleton, image_iff]) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    95
by (dtac fun_cong 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    96
by Auto_tac;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    97
val lemma1 = result();
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
    98
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
    99
Goalw (cmd_defs @ [FP_def, fixedpoint_def, stable_def, constrains_def])
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   100
    "fixedpoint <= FP racts";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   101
by (auto_tac (claset() addIs [ext], simpset()));
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   102
val lemma2 = result();
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   103
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
   104
Goal "FP racts = fixedpoint";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   105
by (rtac ([lemma1,lemma2] MRS equalityI) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   106
qed "FP_fixedpoint";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   107
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   108
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   109
(*If we haven't reached a fixedpoint then there is some edge for which u but
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   110
  not v holds.  Progress will be proved via an ENSURES assertion that the
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   111
  metric will decrease for each suitable edge.  A union over all edges proves
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   112
  a LEADSTO assertion that the metric decreases if we are not at a fixedpoint.
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   113
  *)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   114
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
   115
Goal "Compl fixedpoint = (UN (u,v): edges. {s. s u & ~ s v})";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   116
by (simp_tac (simpset() addsimps
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   117
	      ([Compl_FP, UN_UN_flatten, FP_fixedpoint RS sym, 
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   118
		racts_def, asgt_def])) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   119
by Safe_tac;
5196
1dd4ec921f71 update -> fun_upd
nipkow
parents: 5111
diff changeset
   120
by (rtac fun_upd_idem 1);
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   121
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   122
by (Full_simp_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   123
by (REPEAT (dtac bspec 1 THEN Simp_tac 1));
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   124
by (dtac subsetD 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   125
by (Simp_tac 1);
5196
1dd4ec921f71 update -> fun_upd
nipkow
parents: 5111
diff changeset
   126
by (asm_full_simp_tac (simpset() addsimps [fun_upd_idem_iff]) 1);
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   127
qed "Compl_fixedpoint";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   128
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
   129
Goal "A - fixedpoint = (UN (u,v): edges. A Int {s. s u & ~ s v})";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   130
by (simp_tac (simpset() addsimps [Diff_eq, Compl_fixedpoint]) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   131
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   132
qed "Diff_fixedpoint";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   133
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   134
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   135
(*** Progress ***)
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   136
5111
8f4b72f0c15d Uncurried functions LeadsTo and reach
paulson
parents: 5071
diff changeset
   137
Goalw [metric_def] "~ s x ==> Suc (metric (s(x:=True))) = metric s";
5071
548f398d770b Consequences of the change from [ := ] to ( := ) in theory Update.
nipkow
parents: 5069
diff changeset
   138
by (subgoal_tac "{v. ~ (s(x:=True)) v} = {v. ~ s v} - {x}" 1);
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   139
by Auto_tac;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   140
by (asm_simp_tac (simpset() addsimps [card_Suc_Diff]) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   141
qed "Suc_metric";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   142
5111
8f4b72f0c15d Uncurried functions LeadsTo and reach
paulson
parents: 5071
diff changeset
   143
Goal "~ s x ==> metric (s(x:=True)) < metric s";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   144
by (etac (Suc_metric RS subst) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   145
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   146
qed "metric_less";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   147
AddSIs [metric_less];
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   148
5071
548f398d770b Consequences of the change from [ := ] to ( := ) in theory Update.
nipkow
parents: 5069
diff changeset
   149
Goal "metric (s(y:=s x | s y)) <= metric s";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   150
by (case_tac "s x --> s y" 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   151
by (auto_tac (claset() addIs [less_imp_le],
5196
1dd4ec921f71 update -> fun_upd
nipkow
parents: 5111
diff changeset
   152
	      simpset() addsimps [fun_upd_idem]));
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   153
qed "metric_le";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   154
5111
8f4b72f0c15d Uncurried functions LeadsTo and reach
paulson
parents: 5071
diff changeset
   155
Goal "(u,v): edges ==> \
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   156
\              ensures racts ((metric-``{m}) Int {s. s u & ~ s v})  \
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   157
\                            (metric-``(lessThan m))";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   158
by (ensures_tac "asgt u v" 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   159
by (cut_facts_tac [metric_le] 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   160
by (fast_tac (claset() addSDs [le_imp_less_or_eq]) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   161
qed "edges_ensures";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   162
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
   163
Goal "leadsTo racts ((metric-``{m}) - fixedpoint) (metric-``(lessThan m))";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   164
by (simp_tac (simpset() addsimps [Diff_fixedpoint]) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   165
by (rtac leadsTo_UN 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   166
by (split_all_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   167
by (asm_simp_tac (simpset() addsimps [edges_ensures RS leadsTo_Basis]) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   168
qed "leadsTo_Diff_fixedpoint";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   169
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
   170
Goal "leadsTo racts (metric-``{m}) (metric-``(lessThan m) Un fixedpoint)";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   171
by (rtac (leadsTo_Diff_fixedpoint RS leadsTo_weaken_R RS leadsTo_Diff) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   172
by (ALLGOALS (blast_tac (claset() addIs [subset_imp_leadsTo])));
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   173
qed "leadsTo_Un_fixedpoint";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   174
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   175
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   176
(*Execution in any state leads to a fixedpoint (i.e. can terminate)*)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4896
diff changeset
   177
Goal "leadsTo racts UNIV fixedpoint";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   178
by (rtac lessThan_induct 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   179
by Auto_tac;
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   180
by (rtac leadsTo_Un_fixedpoint 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   181
qed "leadsTo_fixedpoint";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   182
5111
8f4b72f0c15d Uncurried functions LeadsTo and reach
paulson
parents: 5071
diff changeset
   183
Goal "LeadsTo(rinit,racts) UNIV { %v. (init, v) : edges^* }";
4776
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   184
by (stac (fixedpoint_invariant_correct RS sym) 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   185
by (rtac (leadsTo_fixedpoint RS leadsTo_imp_LeadsTo RS LeadsTo_weaken_R) 1); 
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   186
by (cut_facts_tac [reachable_subset_invariant] 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   187
by (Blast_tac 1);
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   188
qed "LeadsTo_correct";
1f9362e769c1 New UNITY theory
paulson
parents:
diff changeset
   189