src/HOL/Hoare/SchorrWaite.thy
author wenzelm
Sat, 05 Jan 2019 17:24:33 +0100
changeset 69597 ff784d5a5bfb
parent 67443 3abf6a722518
child 72806 4fa08e083865
permissions -rw-r--r--
isabelle update -u control_cartouches;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
     1
(*  Title:      HOL/Hoare/SchorrWaite.thy
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
     2
    Author:     Farhad Mehta
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
     3
    Copyright   2003 TUM
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
     4
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
     5
Proof of the Schorr-Waite graph marking algorithm.
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
     6
*)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
     7
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
     8
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 13875
diff changeset
     9
theory SchorrWaite imports HeapSyntax begin
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    10
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
    11
section \<open>Machinery for the Schorr-Waite proof\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    12
36866
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    13
definition
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
    14
  \<comment> \<open>Relations induced by a mapping\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    15
  rel :: "('a \<Rightarrow> 'a ref) \<Rightarrow> ('a \<times> 'a) set"
36866
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    16
  where "rel m = {(x,y). m x = Ref y}"
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    17
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    18
definition
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    19
  relS :: "('a \<Rightarrow> 'a ref) set \<Rightarrow> ('a \<times> 'a) set"
60585
48fdff264eb2 tuned whitespace;
wenzelm
parents: 44890
diff changeset
    20
  where "relS M = (\<Union>m \<in> M. rel m)"
36866
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    21
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    22
definition
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    23
  addrs :: "'a ref set \<Rightarrow> 'a set"
36866
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    24
  where "addrs P = {a. Ref a \<in> P}"
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    25
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    26
definition
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    27
  reachable :: "('a \<times> 'a) set \<Rightarrow> 'a ref set \<Rightarrow> 'a set"
36866
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    28
  where "reachable r P = (r\<^sup>* `` addrs P)"
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    29
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    30
lemmas rel_defs = relS_def rel_def
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    31
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
    32
text \<open>Rewrite rules for relations induced by a mapping\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    33
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    34
lemma self_reachable: "b \<in> B \<Longrightarrow> b \<in> R\<^sup>* `` B"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    35
apply blast
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    36
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    37
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    38
lemma oneStep_reachable: "b \<in> R``B \<Longrightarrow> b \<in> R\<^sup>* `` B"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    39
apply blast
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    40
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    41
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    42
lemma still_reachable: "\<lbrakk>B\<subseteq>Ra\<^sup>*``A; \<forall> (x,y) \<in> Rb-Ra. y\<in> (Ra\<^sup>*``A)\<rbrakk> \<Longrightarrow> Rb\<^sup>* `` B \<subseteq> Ra\<^sup>* `` A "
42154
478bdcea240a tuned proofs;
wenzelm
parents: 39302
diff changeset
    43
apply (clarsimp simp only:Image_iff)
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    44
apply (erule rtrancl_induct)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    45
 apply blast
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    46
apply (subgoal_tac "(y, z) \<in> Ra\<union>(Rb-Ra)")
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    47
 apply (erule UnE)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    48
 apply (auto intro:rtrancl_into_rtrancl)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    49
apply blast
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    50
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    51
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    52
lemma still_reachable_eq: "\<lbrakk> A\<subseteq>Rb\<^sup>*``B; B\<subseteq>Ra\<^sup>*``A; \<forall> (x,y) \<in> Ra-Rb. y \<in>(Rb\<^sup>*``B); \<forall> (x,y) \<in> Rb-Ra. y\<in> (Ra\<^sup>*``A)\<rbrakk> \<Longrightarrow> Ra\<^sup>*``A =  Rb\<^sup>*``B "
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    53
apply (rule equalityI)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    54
 apply (erule still_reachable ,assumption)+
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    55
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    56
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    57
lemma reachable_null: "reachable mS {Null} = {}"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    58
apply (simp add: reachable_def addrs_def)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    59
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    60
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    61
lemma reachable_empty: "reachable mS {} = {}"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    62
apply (simp add: reachable_def addrs_def)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    63
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    64
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    65
lemma reachable_union: "(reachable mS aS \<union> reachable mS bS) = reachable mS (aS \<union> bS)"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    66
apply (simp add: reachable_def rel_defs addrs_def)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    67
apply blast
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    68
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    69
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    70
lemma reachable_union_sym: "reachable r (insert a aS) = (r\<^sup>* `` addrs {a}) \<union> reachable r aS"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    71
apply (simp add: reachable_def rel_defs addrs_def)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    72
apply blast
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    73
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    74
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    75
lemma rel_upd1: "(a,b) \<notin> rel (r(q:=t)) \<Longrightarrow> (a,b) \<in> rel r \<Longrightarrow> a=q"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    76
apply (rule classical)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    77
apply (simp add:rel_defs fun_upd_apply)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    78
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    79
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    80
lemma rel_upd2: "(a,b)  \<notin> rel r \<Longrightarrow> (a,b) \<in> rel (r(q:=t)) \<Longrightarrow> a=q"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    81
apply (rule classical)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    82
apply (simp add:rel_defs fun_upd_apply)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    83
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    84
36866
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    85
definition
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
    86
  \<comment> \<open>Restriction of a relation\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    87
  restr ::"('a \<times> 'a) set \<Rightarrow> ('a \<Rightarrow> bool) \<Rightarrow> ('a \<times> 'a) set"       ("(_/ | _)" [50, 51] 50)
36866
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
    88
  where "restr r m = {(x,y). (x,y) \<in> r \<and> \<not> m x}"
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    89
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
    90
text \<open>Rewrite rules for the restriction of a relation\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    91
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    92
lemma restr_identity[simp]:
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    93
 " (\<forall>x. \<not> m x) \<Longrightarrow> (R |m) = R"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    94
by (auto simp add:restr_def)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    95
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    96
lemma restr_rtrancl[simp]: " \<lbrakk>m l\<rbrakk> \<Longrightarrow> (R | m)\<^sup>* `` {l} = {l}"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    97
by (auto simp add:restr_def elim:converse_rtranclE)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    98
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
    99
lemma [simp]: " \<lbrakk>m l\<rbrakk> \<Longrightarrow> (l,x) \<in> (R | m)\<^sup>* = (l=x)"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   100
by (auto simp add:restr_def elim:converse_rtranclE)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   101
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   102
lemma restr_upd: "((rel (r (q := t)))|(m(q := True))) = ((rel (r))|(m(q := True))) "
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   103
apply (auto simp:restr_def rel_def fun_upd_apply)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   104
apply (rename_tac a b)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   105
apply (case_tac "a=q")
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   106
 apply auto
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   107
done
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   108
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   109
lemma restr_un: "((r \<union> s)|m) = (r|m) \<union> (s|m)"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   110
  by (auto simp add:restr_def)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   111
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   112
lemma rel_upd3: "(a, b) \<notin> (r|(m(q := t))) \<Longrightarrow> (a,b) \<in> (r|m) \<Longrightarrow> a = q "
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   113
apply (rule classical)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   114
apply (simp add:restr_def fun_upd_apply)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   115
done
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   116
36866
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
   117
definition
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   118
  \<comment> \<open>A short form for the stack mapping function for List\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   119
  S :: "('a \<Rightarrow> bool) \<Rightarrow> ('a \<Rightarrow> 'a ref) \<Rightarrow> ('a \<Rightarrow> 'a ref) \<Rightarrow> ('a \<Rightarrow> 'a ref)"
36866
426d5781bb25 modernized specifications;
wenzelm
parents: 32960
diff changeset
   120
  where "S c l r = (\<lambda>x. if c x then r x else l x)"
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   121
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   122
text \<open>Rewrite rules for Lists using S as their mapping\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   123
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   124
lemma [rule_format,simp]:
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   125
 "\<forall>p. a \<notin> set stack \<longrightarrow> List (S c l r) p stack = List (S (c(a:=x)) (l(a:=y)) (r(a:=z))) p stack"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   126
apply(induct_tac stack)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   127
 apply(simp add:fun_upd_apply S_def)+
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   128
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   129
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   130
lemma [rule_format,simp]:
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   131
 "\<forall>p. a \<notin> set stack \<longrightarrow> List (S c l (r(a:=z))) p stack = List (S c l r) p stack"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   132
apply(induct_tac stack)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   133
 apply(simp add:fun_upd_apply S_def)+
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   134
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   135
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   136
lemma [rule_format,simp]:
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   137
 "\<forall>p. a \<notin> set stack \<longrightarrow> List (S c (l(a:=z)) r) p stack = List (S c l r) p stack"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   138
apply(induct_tac stack)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   139
 apply(simp add:fun_upd_apply S_def)+
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   140
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   141
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   142
lemma [rule_format,simp]:
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   143
 "\<forall>p. a \<notin> set stack \<longrightarrow> List (S (c(a:=z)) l r) p stack = List (S c l r) p stack"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   144
apply(induct_tac stack)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   145
 apply(simp add:fun_upd_apply S_def)+
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   146
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   147
38353
d98baa2cf589 modernized specifications;
wenzelm
parents: 36866
diff changeset
   148
primrec
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   149
  \<comment> \<open>Recursive definition of what is means for a the graph/stack structure to be reconstructible\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   150
  stkOk :: "('a \<Rightarrow> bool) \<Rightarrow> ('a \<Rightarrow> 'a ref) \<Rightarrow> ('a \<Rightarrow> 'a ref) \<Rightarrow> ('a \<Rightarrow> 'a ref) \<Rightarrow> ('a \<Rightarrow> 'a ref) \<Rightarrow> 'a ref \<Rightarrow>'a list \<Rightarrow>  bool"
38353
d98baa2cf589 modernized specifications;
wenzelm
parents: 36866
diff changeset
   151
where
d98baa2cf589 modernized specifications;
wenzelm
parents: 36866
diff changeset
   152
  stkOk_nil:  "stkOk c l r iL iR t [] = True"
d98baa2cf589 modernized specifications;
wenzelm
parents: 36866
diff changeset
   153
| stkOk_cons:
d98baa2cf589 modernized specifications;
wenzelm
parents: 36866
diff changeset
   154
    "stkOk c l r iL iR t (p#stk) = (stkOk c l r iL iR (Ref p) (stk) \<and> 
d98baa2cf589 modernized specifications;
wenzelm
parents: 36866
diff changeset
   155
      iL p = (if c p then l p else t) \<and>
d98baa2cf589 modernized specifications;
wenzelm
parents: 36866
diff changeset
   156
      iR p = (if c p then t else r p))"
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   157
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   158
text \<open>Rewrite rules for stkOk\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   159
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   160
lemma [simp]: "\<And>t. \<lbrakk> x \<notin> set xs; Ref x\<noteq>t \<rbrakk> \<Longrightarrow>
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   161
  stkOk (c(x := f)) l r iL iR t xs = stkOk c l r iL iR t xs"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   162
apply (induct xs)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   163
 apply (auto simp:eq_sym_conv)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   164
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   165
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   166
lemma [simp]: "\<And>t. \<lbrakk> x \<notin> set xs; Ref x\<noteq>t \<rbrakk> \<Longrightarrow>
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   167
 stkOk c (l(x := g)) r iL iR t xs = stkOk c l r iL iR t xs"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   168
apply (induct xs)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   169
 apply (auto simp:eq_sym_conv)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   170
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   171
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   172
lemma [simp]: "\<And>t. \<lbrakk> x \<notin> set xs; Ref x\<noteq>t \<rbrakk> \<Longrightarrow>
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   173
 stkOk c l (r(x := g)) iL iR t xs = stkOk c l r iL iR t xs"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   174
apply (induct xs)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   175
 apply (auto simp:eq_sym_conv)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   176
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   177
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   178
lemma stkOk_r_rewrite [simp]: "\<And>x. x \<notin> set xs \<Longrightarrow>
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   179
  stkOk c l (r(x := g)) iL iR (Ref x) xs = stkOk c l r iL iR (Ref x) xs"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   180
apply (induct xs)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   181
 apply (auto simp:eq_sym_conv)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   182
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   183
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   184
lemma [simp]: "\<And>x. x \<notin> set xs \<Longrightarrow>
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   185
 stkOk c (l(x := g)) r iL iR (Ref x) xs = stkOk c l r iL iR (Ref x) xs"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   186
apply (induct xs)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   187
 apply (auto simp:eq_sym_conv)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   188
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   189
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   190
lemma [simp]: "\<And>x. x \<notin> set xs \<Longrightarrow>
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   191
 stkOk (c(x := g)) l r iL iR (Ref x) xs = stkOk c l r iL iR (Ref x) xs"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   192
apply (induct xs)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   193
 apply (auto simp:eq_sym_conv)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   194
done
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   195
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   196
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   197
section\<open>The Schorr-Waite algorithm\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   198
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   199
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   200
theorem SchorrWaiteAlgorithm: 
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   201
"VARS c m l r t p q root
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   202
 {R = reachable (relS {l, r}) {root} \<and> (\<forall>x. \<not> m x) \<and> iR = r \<and> iL = l} 
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   203
 t := root; p := Null;
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   204
 WHILE p \<noteq> Null \<or> t \<noteq> Null \<and> \<not> t^.m
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   205
 INV {\<exists>stack.
67410
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   206
          List (S c l r) p stack \<and>                                      \<comment> \<open>\<open>i1\<close>\<close>
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   207
          (\<forall>x \<in> set stack. m x) \<and>                                       \<comment> \<open>\<open>i2\<close>\<close>
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   208
          R = reachable (relS{l, r}) {t,p} \<and>                            \<comment> \<open>\<open>i3\<close>\<close>
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   209
          (\<forall>x. x \<in> R \<and> \<not>m x \<longrightarrow>                                         \<comment> \<open>\<open>i4\<close>\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   210
                 x \<in> reachable (relS{l,r}|m) ({t}\<union>set(map r stack))) \<and>
67410
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   211
          (\<forall>x. m x \<longrightarrow> x \<in> R) \<and>                                         \<comment> \<open>\<open>i5\<close>\<close>
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   212
          (\<forall>x. x \<notin> set stack \<longrightarrow> r x = iR x \<and> l x = iL x) \<and>             \<comment> \<open>\<open>i6\<close>\<close>
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   213
          (stkOk c l r iL iR t stack)                                   \<comment> \<open>\<open>i7\<close>\<close>}
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   214
 DO IF t = Null \<or> t^.m
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   215
      THEN IF p^.c
67410
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   216
               THEN q := t; t := p; p := p^.r; t^.r := q                \<comment> \<open>\<open>pop\<close>\<close>
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   217
               ELSE q := t; t := p^.r; p^.r := p^.l;                    \<comment> \<open>\<open>swing\<close>\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   218
                        p^.l := q; p^.c := True          FI    
67410
64d928bacddd prefer formal comments;
wenzelm
parents: 62042
diff changeset
   219
      ELSE q := p; p := t; t := t^.l; p^.l := q;                        \<comment> \<open>\<open>push\<close>\<close>
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   220
               p^.m := True; p^.c := False            FI       OD
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   221
 {(\<forall>x. (x \<in> R) = m x) \<and> (r = iR \<and> l = iL) }"
13875
12997e3ddd8d *** empty log message ***
nipkow
parents: 13820
diff changeset
   222
  (is "VARS c m l r t p q root {?Pre c m l r root} (?c1; ?c2; ?c3) {?Post c m l r}")
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   223
proof (vcg)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   224
  let "While {(c, m, l, r, t, p, q, root). ?whileB m t p}
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   225
    {(c, m, l, r, t, p, q, root). ?inv c m l r t p} ?body" = ?c3
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   226
  {
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   227
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   228
    fix c m l r t p q root
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   229
    assume "?Pre c m l r root"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   230
    thus "?inv c m l r root Null"  by (auto simp add: reachable_def addrs_def)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   231
  next
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   232
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   233
    fix c m l r t p q
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   234
    let "\<exists>stack. ?Inv stack"  =  "?inv c m l r t p"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   235
    assume a: "?inv c m l r t p \<and> \<not>(p \<noteq> Null \<or> t \<noteq> Null \<and> \<not> t^.m)"  
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   236
    then obtain stack where inv: "?Inv stack" by blast
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   237
    from a have pNull: "p = Null" and tDisj: "t=Null \<or> (t\<noteq>Null \<and> t^.m )" by auto
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   238
    let "?I1 \<and> _ \<and> _ \<and> ?I4 \<and> ?I5 \<and> ?I6 \<and> _"  =  "?Inv stack"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   239
    from inv have i1: "?I1" and i4: "?I4" and i5: "?I5" and i6: "?I6" by simp+
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   240
    from pNull i1 have stackEmpty: "stack = []" by simp
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   241
    from tDisj i4 have RisMarked[rule_format]: "\<forall>x.  x \<in> R \<longrightarrow> m x"  by(auto simp: reachable_def addrs_def stackEmpty)
39302
d7728f65b353 renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
nipkow
parents: 39198
diff changeset
   242
    from i5 i6 show "(\<forall>x.(x \<in> R) = m x) \<and> r = iR \<and> l = iL"  by(auto simp: stackEmpty fun_eq_iff intro:RisMarked)
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   243
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   244
  next   
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   245
      fix c m l r t p q root
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   246
      let "\<exists>stack. ?Inv stack"  =  "?inv c m l r t p"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   247
      let "\<exists>stack. ?popInv stack"  =  "?inv c m l (r(p \<rightarrow> t)) p (p^.r)"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   248
      let "\<exists>stack. ?swInv stack"  =
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   249
        "?inv (c(p \<rightarrow> True)) m (l(p \<rightarrow> t)) (r(p \<rightarrow> p^.l)) (p^.r) p"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   250
      let "\<exists>stack. ?puInv stack"  =
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   251
        "?inv (c(t \<rightarrow> False)) (m(t \<rightarrow> True)) (l(t \<rightarrow> p)) r (t^.l) t"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   252
      let "?ifB1"  =  "(t = Null \<or> t^.m)"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   253
      let "?ifB2"  =  "p^.c" 
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   254
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   255
      assume "(\<exists>stack.?Inv stack) \<and> (p \<noteq> Null \<or> t \<noteq> Null \<and> \<not> t^.m)" (is "_ \<and> ?whileB")
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   256
      then obtain stack where inv: "?Inv stack" and whileB: "?whileB" by blast
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   257
      let "?I1 \<and> ?I2 \<and> ?I3 \<and> ?I4 \<and> ?I5 \<and> ?I6 \<and> ?I7" = "?Inv stack"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   258
      from inv have i1: "?I1" and i2: "?I2" and i3: "?I3" and i4: "?I4"
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   259
                  and i5: "?I5" and i6: "?I6" and i7: "?I7" by simp+        
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   260
      have stackDist: "distinct (stack)" using i1 by (rule List_distinct)
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   261
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   262
      show "(?ifB1 \<longrightarrow> (?ifB2 \<longrightarrow> (\<exists>stack.?popInv stack)) \<and> 
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   263
                            (\<not>?ifB2 \<longrightarrow> (\<exists>stack.?swInv stack)) ) \<and>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   264
              (\<not>?ifB1 \<longrightarrow> (\<exists>stack.?puInv stack))"
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   265
      proof - 
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   266
        {
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   267
          assume ifB1: "t = Null \<or> t^.m" and ifB2: "p^.c"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   268
          from ifB1 whileB have pNotNull: "p \<noteq> Null" by auto
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   269
          then obtain addr_p where addr_p_eq: "p = Ref addr_p" by auto
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   270
          with i1 obtain stack_tl where stack_eq: "stack = (addr p) # stack_tl"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   271
            by auto
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   272
          with i2 have m_addr_p: "p^.m" by auto
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   273
          have stackDist: "distinct (stack)" using i1 by (rule List_distinct)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   274
          from stack_eq stackDist have p_notin_stack_tl: "addr p \<notin> set stack_tl" by simp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   275
          let "?poI1\<and> ?poI2\<and> ?poI3\<and> ?poI4\<and> ?poI5\<and> ?poI6\<and> ?poI7" = "?popInv stack_tl"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   276
          have "?popInv stack_tl"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   277
          proof -
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   278
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   279
            \<comment> \<open>List property is maintained:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   280
            from i1 p_notin_stack_tl ifB2
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   281
            have poI1: "List (S c l (r(p \<rightarrow> t))) (p^.r) stack_tl" 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   282
              by(simp add: addr_p_eq stack_eq, simp add: S_def)
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   283
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   284
            moreover
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   285
            \<comment> \<open>Everything on the stack is marked:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   286
            from i2 have poI2: "\<forall> x \<in> set stack_tl. m x" by (simp add:stack_eq)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   287
            moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   288
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   289
            \<comment> \<open>Everything is still reachable:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   290
            let "(R = reachable ?Ra ?A)" = "?I3"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   291
            let "?Rb" = "(relS {l, r(p \<rightarrow> t)})"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   292
            let "?B" = "{p, p^.r}"
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   293
            \<comment> \<open>Our goal is \<open>R = reachable ?Rb ?B\<close>.\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   294
            have "?Ra\<^sup>* `` addrs ?A = ?Rb\<^sup>* `` addrs ?B" (is "?L = ?R")
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   295
            proof
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   296
              show "?L \<subseteq> ?R"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   297
              proof (rule still_reachable)
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   298
                show "addrs ?A \<subseteq> ?Rb\<^sup>* `` addrs ?B" by(fastforce simp:addrs_def relS_def rel_def addr_p_eq 
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   299
                     intro:oneStep_reachable Image_iff[THEN iffD2])
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   300
                show "\<forall>(x,y) \<in> ?Ra-?Rb. y \<in> (?Rb\<^sup>* `` addrs ?B)" by (clarsimp simp:relS_def) 
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   301
                     (fastforce simp add:rel_def Image_iff addrs_def dest:rel_upd1)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   302
              qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   303
              show "?R \<subseteq> ?L"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   304
              proof (rule still_reachable)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   305
                show "addrs ?B \<subseteq> ?Ra\<^sup>* `` addrs ?A"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   306
                  by(fastforce simp:addrs_def rel_defs addr_p_eq 
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   307
                      intro:oneStep_reachable Image_iff[THEN iffD2])
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   308
              next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   309
                show "\<forall>(x, y)\<in>?Rb-?Ra. y\<in>(?Ra\<^sup>*``addrs ?A)"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   310
                  by (clarsimp simp:relS_def) 
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   311
                     (fastforce simp add:rel_def Image_iff addrs_def dest:rel_upd2)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   312
              qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   313
            qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   314
            with i3 have poI3: "R = reachable ?Rb ?B"  by (simp add:reachable_def) 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   315
            moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   316
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   317
            \<comment> \<open>If it is reachable and not marked, it is still reachable using...\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   318
            let "\<forall>x. x \<in> R \<and> \<not> m x \<longrightarrow> x \<in> reachable ?Ra ?A"  =  ?I4        
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   319
            let "?Rb" = "relS {l, r(p \<rightarrow> t)} | m"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   320
            let "?B" = "{p} \<union> set (map (r(p \<rightarrow> t)) stack_tl)"
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   321
            \<comment> \<open>Our goal is \<open>\<forall>x. x \<in> R \<and> \<not> m x \<longrightarrow> x \<in> reachable ?Rb ?B\<close>.\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   322
            let ?T = "{t, p^.r}"
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   323
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   324
            have "?Ra\<^sup>* `` addrs ?A \<subseteq> ?Rb\<^sup>* `` (addrs ?B \<union> addrs ?T)"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   325
            proof (rule still_reachable)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   326
              have rewrite: "\<forall>s\<in>set stack_tl. (r(p \<rightarrow> t)) s = r s"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   327
                by (auto simp add:p_notin_stack_tl intro:fun_upd_other) 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   328
              show "addrs ?A \<subseteq> ?Rb\<^sup>* `` (addrs ?B \<union> addrs ?T)"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   329
                by (fastforce cong:map_cong simp:stack_eq addrs_def rewrite intro:self_reachable)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   330
              show "\<forall>(x, y)\<in>?Ra-?Rb. y\<in>(?Rb\<^sup>*``(addrs ?B \<union> addrs ?T))"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   331
                by (clarsimp simp:restr_def relS_def) 
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   332
                  (fastforce simp add:rel_def Image_iff addrs_def dest:rel_upd1)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   333
            qed
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   334
            \<comment> \<open>We now bring a term from the right to the left of the subset relation.\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   335
            hence subset: "?Ra\<^sup>* `` addrs ?A - ?Rb\<^sup>* `` addrs ?T \<subseteq> ?Rb\<^sup>* `` addrs ?B"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   336
              by blast
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   337
            have poI4: "\<forall>x. x \<in> R \<and> \<not> m x \<longrightarrow> x \<in> reachable ?Rb ?B"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   338
            proof (rule allI, rule impI)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   339
              fix x
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   340
              assume a: "x \<in> R \<and> \<not> m x"
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67443
diff changeset
   341
              \<comment> \<open>First, a disjunction on \<^term>\<open>p^.r\<close> used later in the proof\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   342
              have pDisj:"p^.r = Null \<or> (p^.r \<noteq> Null \<and> p^.r^.m)" using poI1 poI2 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   343
                by auto
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67443
diff changeset
   344
              \<comment> \<open>\<^term>\<open>x\<close> belongs to the left hand side of @{thm[source] subset}:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   345
              have incl: "x \<in> ?Ra\<^sup>*``addrs ?A" using  a i4 by (simp only:reachable_def, clarsimp)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   346
              have excl: "x \<notin> ?Rb\<^sup>*`` addrs ?T" using pDisj ifB1 a by (auto simp add:addrs_def)
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   347
              \<comment> \<open>And therefore also belongs to the right hand side of @{thm[source]subset},\<close>
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   348
              \<comment> \<open>which corresponds to our goal.\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   349
              from incl excl subset  show "x \<in> reachable ?Rb ?B" by (auto simp add:reachable_def)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   350
            qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   351
            moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   352
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   353
            \<comment> \<open>If it is marked, then it is reachable\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   354
            from i5 have poI5: "\<forall>x. m x \<longrightarrow> x \<in> R" .
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   355
            moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   356
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67443
diff changeset
   357
            \<comment> \<open>If it is not on the stack, then its \<^term>\<open>l\<close> and \<^term>\<open>r\<close> fields are unchanged\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   358
            from i7 i6 ifB2 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   359
            have poI6: "\<forall>x. x \<notin> set stack_tl \<longrightarrow> (r(p \<rightarrow> t)) x = iR x \<and> l x = iL x" 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   360
              by(auto simp: addr_p_eq stack_eq fun_upd_apply)
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   361
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   362
            moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   363
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67443
diff changeset
   364
            \<comment> \<open>If it is on the stack, then its \<^term>\<open>l\<close> and \<^term>\<open>r\<close> fields can be reconstructed\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   365
            from p_notin_stack_tl i7 have poI7: "stkOk c l (r(p \<rightarrow> t)) iL iR p stack_tl"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   366
              by (clarsimp simp:stack_eq addr_p_eq)
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   367
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   368
            ultimately show "?popInv stack_tl" by simp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   369
          qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   370
          hence "\<exists>stack. ?popInv stack" ..
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   371
        }
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   372
        moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   373
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   374
        \<comment> \<open>Proofs of the Swing and Push arm follow.\<close>
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   375
        \<comment> \<open>Since they are in principle simmilar to the Pop arm proof,\<close>
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   376
        \<comment> \<open>we show fewer comments and use frequent pattern matching.\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   377
        {
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   378
          \<comment> \<open>Swing arm\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   379
          assume ifB1: "?ifB1" and nifB2: "\<not>?ifB2"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   380
          from ifB1 whileB have pNotNull: "p \<noteq> Null" by clarsimp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   381
          then obtain addr_p where addr_p_eq: "p = Ref addr_p" by clarsimp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   382
          with i1 obtain stack_tl where stack_eq: "stack = (addr p) # stack_tl" by clarsimp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   383
          with i2 have m_addr_p: "p^.m" by clarsimp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   384
          from stack_eq stackDist have p_notin_stack_tl: "(addr p) \<notin> set stack_tl"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   385
            by simp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   386
          let "?swI1\<and>?swI2\<and>?swI3\<and>?swI4\<and>?swI5\<and>?swI6\<and>?swI7" = "?swInv stack"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   387
          have "?swInv stack"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   388
          proof -
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   389
            
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   390
            \<comment> \<open>List property is maintained:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   391
            from i1 p_notin_stack_tl nifB2
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   392
            have swI1: "?swI1"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   393
              by (simp add:addr_p_eq stack_eq, simp add:S_def)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   394
            moreover
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   395
            
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   396
            \<comment> \<open>Everything on the stack is marked:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   397
            from i2
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   398
            have swI2: "?swI2" .
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   399
            moreover
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   400
            
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   401
            \<comment> \<open>Everything is still reachable:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   402
            let "R = reachable ?Ra ?A" = "?I3"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   403
            let "R = reachable ?Rb ?B" = "?swI3"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   404
            have "?Ra\<^sup>* `` addrs ?A = ?Rb\<^sup>* `` addrs ?B"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   405
            proof (rule still_reachable_eq)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   406
              show "addrs ?A \<subseteq> ?Rb\<^sup>* `` addrs ?B"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   407
                by(fastforce simp:addrs_def rel_defs addr_p_eq intro:oneStep_reachable Image_iff[THEN iffD2])
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   408
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   409
              show "addrs ?B \<subseteq> ?Ra\<^sup>* `` addrs ?A"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   410
                by(fastforce simp:addrs_def rel_defs addr_p_eq intro:oneStep_reachable Image_iff[THEN iffD2])
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   411
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   412
              show "\<forall>(x, y)\<in>?Ra-?Rb. y\<in>(?Rb\<^sup>*``addrs ?B)"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   413
                by (clarsimp simp:relS_def) (fastforce simp add:rel_def Image_iff addrs_def fun_upd_apply dest:rel_upd1)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   414
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   415
              show "\<forall>(x, y)\<in>?Rb-?Ra. y\<in>(?Ra\<^sup>*``addrs ?A)"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   416
                by (clarsimp simp:relS_def) (fastforce simp add:rel_def Image_iff addrs_def fun_upd_apply dest:rel_upd2)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   417
            qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   418
            with i3
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   419
            have swI3: "?swI3" by (simp add:reachable_def) 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   420
            moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   421
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   422
            \<comment> \<open>If it is reachable and not marked, it is still reachable using...\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   423
            let "\<forall>x. x \<in> R \<and> \<not> m x \<longrightarrow> x \<in> reachable ?Ra ?A" = ?I4
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   424
            let "\<forall>x. x \<in> R \<and> \<not> m x \<longrightarrow> x \<in> reachable ?Rb ?B" = ?swI4
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   425
            let ?T = "{t}"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   426
            have "?Ra\<^sup>*``addrs ?A \<subseteq> ?Rb\<^sup>*``(addrs ?B \<union> addrs ?T)"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   427
            proof (rule still_reachable)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   428
              have rewrite: "(\<forall>s\<in>set stack_tl. (r(addr p := l(addr p))) s = r s)"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   429
                by (auto simp add:p_notin_stack_tl intro:fun_upd_other)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   430
              show "addrs ?A \<subseteq> ?Rb\<^sup>* `` (addrs ?B \<union> addrs ?T)"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   431
                by (fastforce cong:map_cong simp:stack_eq addrs_def rewrite intro:self_reachable)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   432
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   433
              show "\<forall>(x, y)\<in>?Ra-?Rb. y\<in>(?Rb\<^sup>*``(addrs ?B \<union> addrs ?T))"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   434
                by (clarsimp simp:relS_def restr_def) (fastforce simp add:rel_def Image_iff addrs_def fun_upd_apply dest:rel_upd1)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   435
            qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   436
            then have subset: "?Ra\<^sup>*``addrs ?A - ?Rb\<^sup>*``addrs ?T \<subseteq> ?Rb\<^sup>*``addrs ?B"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   437
              by blast
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   438
            have ?swI4
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   439
            proof (rule allI, rule impI)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   440
              fix x
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   441
              assume a: "x \<in> R \<and>\<not> m x"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   442
              with i4 addr_p_eq stack_eq  have inc: "x \<in> ?Ra\<^sup>*``addrs ?A" 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   443
                by (simp only:reachable_def, clarsimp)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   444
              with ifB1 a 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   445
              have exc: "x \<notin> ?Rb\<^sup>*`` addrs ?T" 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   446
                by (auto simp add:addrs_def)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   447
              from inc exc subset  show "x \<in> reachable ?Rb ?B" 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   448
                by (auto simp add:reachable_def)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   449
            qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   450
            moreover
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   451
            
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   452
            \<comment> \<open>If it is marked, then it is reachable\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   453
            from i5
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   454
            have "?swI5" .
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   455
            moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   456
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67443
diff changeset
   457
            \<comment> \<open>If it is not on the stack, then its \<^term>\<open>l\<close> and \<^term>\<open>r\<close> fields are unchanged\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   458
            from i6 stack_eq
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   459
            have "?swI6"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   460
              by clarsimp           
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   461
            moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   462
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67443
diff changeset
   463
            \<comment> \<open>If it is on the stack, then its \<^term>\<open>l\<close> and \<^term>\<open>r\<close> fields can be reconstructed\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   464
            from stackDist i7 nifB2 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   465
            have "?swI7"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   466
              by (clarsimp simp:addr_p_eq stack_eq)
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   467
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   468
            ultimately show ?thesis by auto
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   469
          qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   470
          then have "\<exists>stack. ?swInv stack" by blast
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   471
        }
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   472
        moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   473
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   474
        {
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   475
          \<comment> \<open>Push arm\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   476
          assume nifB1: "\<not>?ifB1"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   477
          from nifB1 whileB have tNotNull: "t \<noteq> Null" by clarsimp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   478
          then obtain addr_t where addr_t_eq: "t = Ref addr_t" by clarsimp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   479
          with i1 obtain new_stack where new_stack_eq: "new_stack = (addr t) # stack" by clarsimp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   480
          from tNotNull nifB1 have n_m_addr_t: "\<not> (t^.m)" by clarsimp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   481
          with i2 have t_notin_stack: "(addr t) \<notin> set stack" by blast
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   482
          let "?puI1\<and>?puI2\<and>?puI3\<and>?puI4\<and>?puI5\<and>?puI6\<and>?puI7" = "?puInv new_stack"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   483
          have "?puInv new_stack"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   484
          proof -
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   485
            
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   486
            \<comment> \<open>List property is maintained:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   487
            from i1 t_notin_stack
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   488
            have puI1: "?puI1"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   489
              by (simp add:addr_t_eq new_stack_eq, simp add:S_def)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   490
            moreover
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   491
            
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   492
            \<comment> \<open>Everything on the stack is marked:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   493
            from i2
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   494
            have puI2: "?puI2" 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   495
              by (simp add:new_stack_eq fun_upd_apply)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   496
            moreover
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   497
            
62042
6c6ccf573479 isabelle update_cartouches -c -t;
wenzelm
parents: 60585
diff changeset
   498
            \<comment> \<open>Everything is still reachable:\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   499
            let "R = reachable ?Ra ?A" = "?I3"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   500
            let "R = reachable ?Rb ?B" = "?puI3"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   501
            have "?Ra\<^sup>* `` addrs ?A = ?Rb\<^sup>* `` addrs ?B"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   502
            proof (rule still_reachable_eq)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   503
              show "addrs ?A \<subseteq> ?Rb\<^sup>* `` addrs ?B"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   504
                by(fastforce simp:addrs_def rel_defs addr_t_eq intro:oneStep_reachable Image_iff[THEN iffD2])
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   505
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   506
              show "addrs ?B \<subseteq> ?Ra\<^sup>* `` addrs ?A"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   507
                by(fastforce simp:addrs_def rel_defs addr_t_eq intro:oneStep_reachable Image_iff[THEN iffD2])
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   508
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   509
              show "\<forall>(x, y)\<in>?Ra-?Rb. y\<in>(?Rb\<^sup>*``addrs ?B)"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   510
                by (clarsimp simp:relS_def) (fastforce simp add:rel_def Image_iff addrs_def dest:rel_upd1)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   511
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   512
              show "\<forall>(x, y)\<in>?Rb-?Ra. y\<in>(?Ra\<^sup>*``addrs ?A)"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   513
                by (clarsimp simp:relS_def) (fastforce simp add:rel_def Image_iff addrs_def fun_upd_apply dest:rel_upd2)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   514
            qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   515
            with i3
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   516
            have puI3: "?puI3" by (simp add:reachable_def) 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   517
            moreover
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   518
            
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   519
            \<comment> \<open>If it is reachable and not marked, it is still reachable using...\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   520
            let "\<forall>x. x \<in> R \<and> \<not> m x \<longrightarrow> x \<in> reachable ?Ra ?A" = ?I4
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   521
            let "\<forall>x. x \<in> R \<and> \<not> ?new_m x \<longrightarrow> x \<in> reachable ?Rb ?B" = ?puI4
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   522
            let ?T = "{t}"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   523
            have "?Ra\<^sup>*``addrs ?A \<subseteq> ?Rb\<^sup>*``(addrs ?B \<union> addrs ?T)"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   524
            proof (rule still_reachable)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   525
              show "addrs ?A \<subseteq> ?Rb\<^sup>* `` (addrs ?B \<union> addrs ?T)"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   526
                by (fastforce simp:new_stack_eq addrs_def intro:self_reachable)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   527
            next
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   528
              show "\<forall>(x, y)\<in>?Ra-?Rb. y\<in>(?Rb\<^sup>*``(addrs ?B \<union> addrs ?T))"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   529
                by (clarsimp simp:relS_def new_stack_eq restr_un restr_upd) 
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   530
                   (fastforce simp add:rel_def Image_iff restr_def addrs_def fun_upd_apply addr_t_eq dest:rel_upd3)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   531
            qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   532
            then have subset: "?Ra\<^sup>*``addrs ?A - ?Rb\<^sup>*``addrs ?T \<subseteq> ?Rb\<^sup>*``addrs ?B"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   533
              by blast
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   534
            have ?puI4
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   535
            proof (rule allI, rule impI)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   536
              fix x
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   537
              assume a: "x \<in> R \<and> \<not> ?new_m x"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   538
              have xDisj: "x=(addr t) \<or> x\<noteq>(addr t)" by simp
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   539
              with i4 a have inc: "x \<in> ?Ra\<^sup>*``addrs ?A"
44890
22f665a2e91c new fastforce replacing fastsimp - less confusing name
nipkow
parents: 42154
diff changeset
   540
                by (fastforce simp:addr_t_eq addrs_def reachable_def intro:self_reachable)
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   541
              have exc: "x \<notin> ?Rb\<^sup>*`` addrs ?T"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   542
                using xDisj a n_m_addr_t
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   543
                by (clarsimp simp add:addrs_def addr_t_eq) 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   544
              from inc exc subset  show "x \<in> reachable ?Rb ?B" 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   545
                by (auto simp add:reachable_def)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   546
            qed  
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   547
            moreover
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   548
            
67443
3abf6a722518 standardized towards new-style formal comments: isabelle update_comments;
wenzelm
parents: 67410
diff changeset
   549
            \<comment> \<open>If it is marked, then it is reachable\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   550
            from i5
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   551
            have "?puI5"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   552
              by (auto simp:addrs_def i3 reachable_def addr_t_eq fun_upd_apply intro:self_reachable)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   553
            moreover
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   554
            
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67443
diff changeset
   555
            \<comment> \<open>If it is not on the stack, then its \<^term>\<open>l\<close> and \<^term>\<open>r\<close> fields are unchanged\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   556
            from i6 
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   557
            have "?puI6"
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   558
              by (simp add:new_stack_eq)
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   559
            moreover
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   560
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67443
diff changeset
   561
            \<comment> \<open>If it is on the stack, then its \<^term>\<open>l\<close> and \<^term>\<open>r\<close> fields can be reconstructed\<close>
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   562
            from stackDist i6 t_notin_stack i7
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   563
            have "?puI7" by (clarsimp simp:addr_t_eq new_stack_eq)
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   564
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   565
            ultimately show ?thesis by auto
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   566
          qed
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   567
          then have "\<exists>stack. ?puInv stack" by blast
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   568
32960
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   569
        }
69916a850301 eliminated hard tabulators, guessing at each author's individual tab-width;
wenzelm
parents: 16417
diff changeset
   570
        ultimately show ?thesis by blast
13820
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   571
      qed
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   572
    }
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   573
  qed
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   574
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   575
end
87a8ab465b29 Proof of the Schorr-Waite graph marking algorithm.
mehta
parents:
diff changeset
   576