author | paulson <lp15@cam.ac.uk> |
Sat, 04 Dec 2021 20:30:16 +0000 | |
changeset 74878 | 0263787a06b4 |
parent 74723 | f05c73bf5968 |
child 80914 | d97fdabd9e2b |
permissions | -rw-r--r-- |
41959 | 1 |
(* Title: HOL/Hoare/Hoare_Logic.thy |
5646 | 2 |
Author: Leonor Prensa Nieto & Tobias Nipkow |
3 |
Copyright 1998 TUM |
|
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
4 |
Author: Walter Guttmann (extension to total-correctness proofs) |
1335 | 5 |
*) |
6 |
||
72990 | 7 |
section \<open>Hoare logic\<close> |
8 |
||
9 |
theory Hoare_Logic |
|
10 |
imports Hoare_Syntax Hoare_Tac |
|
11 |
begin |
|
12 |
||
13 |
subsection \<open>Sugared semantic embedding of Hoare logic\<close> |
|
72987
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
14 |
|
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
15 |
text \<open> |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
16 |
Strictly speaking a shallow embedding (as implemented by Norbert Galm |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
17 |
following Mike Gordon) would suffice. Maybe the datatype com comes in useful |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
18 |
later. |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
19 |
\<close> |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
20 |
|
42174 | 21 |
type_synonym 'a bexp = "'a set" |
22 |
type_synonym 'a assn = "'a set" |
|
5646 | 23 |
|
58310 | 24 |
datatype 'a com = |
58305
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
55660
diff
changeset
|
25 |
Basic "'a \<Rightarrow> 'a" |
72987
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
26 |
| Seq "'a com" "'a com" |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
27 |
| Cond "'a bexp" "'a com" "'a com" |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
28 |
| While "'a bexp" "'a com" |
35113 | 29 |
|
35054 | 30 |
abbreviation annskip ("SKIP") where "SKIP == Basic id" |
5646 | 31 |
|
42174 | 32 |
type_synonym 'a sem = "'a => 'a => bool" |
5646 | 33 |
|
36643 | 34 |
inductive Sem :: "'a com \<Rightarrow> 'a sem" |
35 |
where |
|
36 |
"Sem (Basic f) s (f s)" |
|
72987
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
37 |
| "Sem c1 s s'' \<Longrightarrow> Sem c2 s'' s' \<Longrightarrow> Sem (Seq c1 c2) s s'" |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
38 |
| "s \<in> b \<Longrightarrow> Sem c1 s s' \<Longrightarrow> Sem (Cond b c1 c2) s s'" |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
39 |
| "s \<notin> b \<Longrightarrow> Sem c2 s s' \<Longrightarrow> Sem (Cond b c1 c2) s s'" |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
40 |
| "s \<notin> b \<Longrightarrow> Sem (While b c) s s" |
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
41 |
| "s \<in> b \<Longrightarrow> Sem c s s'' \<Longrightarrow> Sem (While b c) s'' s' \<Longrightarrow> |
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
42 |
Sem (While b c) s s'" |
5646 | 43 |
|
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
44 |
definition Valid :: "'a bexp \<Rightarrow> 'a com \<Rightarrow> 'a anno \<Rightarrow> 'a bexp \<Rightarrow> bool" |
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
45 |
where "Valid p c a q \<equiv> \<forall>s s'. Sem c s s' \<longrightarrow> s \<in> p \<longrightarrow> s' \<in> q" |
72987
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
46 |
|
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
47 |
definition ValidTC :: "'a bexp \<Rightarrow> 'a com \<Rightarrow> 'a anno \<Rightarrow> 'a bexp \<Rightarrow> bool" |
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
48 |
where "ValidTC p c a q \<equiv> \<forall>s. s \<in> p \<longrightarrow> (\<exists>t. Sem c s t \<and> t \<in> q)" |
72987
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
49 |
|
36643 | 50 |
inductive_cases [elim!]: |
72987
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
51 |
"Sem (Basic f) s s'" "Sem (Seq c1 c2) s s'" |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
52 |
"Sem (Cond b c1 c2) s s'" |
5646 | 53 |
|
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
54 |
lemma Sem_deterministic: |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
55 |
assumes "Sem c s s1" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
56 |
and "Sem c s s2" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
57 |
shows "s1 = s2" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
58 |
proof - |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
59 |
have "Sem c s s1 \<Longrightarrow> (\<forall>s2. Sem c s s2 \<longrightarrow> s1 = s2)" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
60 |
by (induct rule: Sem.induct) (subst Sem.simps, blast)+ |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
61 |
thus ?thesis |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
62 |
using assms by simp |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
63 |
qed |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
64 |
|
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
65 |
lemma tc_implies_pc: |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
66 |
"ValidTC p c a q \<Longrightarrow> Valid p c a q" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
67 |
by (metis Sem_deterministic Valid_def ValidTC_def) |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
68 |
|
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
69 |
lemma tc_extract_function: |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
70 |
"ValidTC p c a q \<Longrightarrow> \<exists>f . \<forall>s . s \<in> p \<longrightarrow> f s \<in> q" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
71 |
by (metis ValidTC_def) |
5007 | 72 |
|
13682 | 73 |
|
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
74 |
lemma SkipRule: "p \<subseteq> q \<Longrightarrow> Valid p (Basic id) a q" |
13857 | 75 |
by (auto simp:Valid_def) |
76 |
||
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
77 |
lemma BasicRule: "p \<subseteq> {s. f s \<in> q} \<Longrightarrow> Valid p (Basic f) a q" |
13857 | 78 |
by (auto simp:Valid_def) |
79 |
||
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
80 |
lemma SeqRule: "Valid P c1 a1 Q \<Longrightarrow> Valid Q c2 a2 R \<Longrightarrow> Valid P (Seq c1 c2) (Aseq a1 a2) R" |
13857 | 81 |
by (auto simp:Valid_def) |
82 |
||
83 |
lemma CondRule: |
|
84 |
"p \<subseteq> {s. (s \<in> b \<longrightarrow> s \<in> w) \<and> (s \<notin> b \<longrightarrow> s \<in> w')} |
|
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
85 |
\<Longrightarrow> Valid w c1 a1 q \<Longrightarrow> Valid w' c2 a2 q \<Longrightarrow> Valid p (Cond b c1 c2) (Acond a1 a2) q" |
13857 | 86 |
by (auto simp:Valid_def) |
87 |
||
36643 | 88 |
lemma While_aux: |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
89 |
assumes "Sem (While b c) s s'" |
36643 | 90 |
shows "\<forall>s s'. Sem c s s' \<longrightarrow> s \<in> I \<and> s \<in> b \<longrightarrow> s' \<in> I \<Longrightarrow> |
91 |
s \<in> I \<Longrightarrow> s' \<in> I \<and> s' \<notin> b" |
|
92 |
using assms |
|
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
93 |
by (induct "While b c" s s') auto |
13857 | 94 |
|
95 |
lemma WhileRule: |
|
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
96 |
"p \<subseteq> i \<Longrightarrow> Valid (i \<inter> b) c (A 0) i \<Longrightarrow> i \<inter> (-b) \<subseteq> q \<Longrightarrow> Valid p (While b c) (Awhile i v A) q" |
13857 | 97 |
apply (clarsimp simp:Valid_def) |
36643 | 98 |
apply(drule While_aux) |
99 |
apply assumption |
|
13857 | 100 |
apply blast |
101 |
apply blast |
|
102 |
done |
|
103 |
||
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
104 |
lemma SkipRuleTC: |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
105 |
assumes "p \<subseteq> q" |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
106 |
shows "ValidTC p (Basic id) a q" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
107 |
by (metis assms Sem.intros(1) ValidTC_def id_apply subsetD) |
13857 | 108 |
|
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
109 |
lemma BasicRuleTC: |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
110 |
assumes "p \<subseteq> {s. f s \<in> q}" |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
111 |
shows "ValidTC p (Basic f) a q" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
112 |
by (metis assms Ball_Collect Sem.intros(1) ValidTC_def) |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
113 |
|
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
114 |
lemma SeqRuleTC: |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
115 |
assumes "ValidTC p c1 a1 q" |
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
116 |
and "ValidTC q c2 a2 r" |
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
117 |
shows "ValidTC p (Seq c1 c2) (Aseq a1 a2) r" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
118 |
by (meson assms Sem.intros(2) ValidTC_def) |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
119 |
|
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
120 |
lemma CondRuleTC: |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
121 |
assumes "p \<subseteq> {s. (s \<in> b \<longrightarrow> s \<in> w) \<and> (s \<notin> b \<longrightarrow> s \<in> w')}" |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
122 |
and "ValidTC w c1 a1 q" |
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
123 |
and "ValidTC w' c2 a2 q" |
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
124 |
shows "ValidTC p (Cond b c1 c2) (Acond a1 a2) q" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
125 |
proof (unfold ValidTC_def, rule allI) |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
126 |
fix s |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
127 |
show "s \<in> p \<longrightarrow> (\<exists>t . Sem (Cond b c1 c2) s t \<and> t \<in> q)" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
128 |
apply (cases "s \<in> b") |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
129 |
apply (metis (mono_tags, lifting) assms(1,2) Ball_Collect Sem.intros(3) ValidTC_def) |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
130 |
by (metis (mono_tags, lifting) assms(1,3) Ball_Collect Sem.intros(4) ValidTC_def) |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
131 |
qed |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
132 |
|
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
133 |
lemma WhileRuleTC: |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
134 |
assumes "p \<subseteq> i" |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
135 |
and "\<And>n::nat . ValidTC (i \<inter> b \<inter> {s . v s = n}) c (A n) (i \<inter> {s . v s < n})" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
136 |
and "i \<inter> uminus b \<subseteq> q" |
74723 | 137 |
shows "ValidTC p (While b c) (Awhile i v (\<lambda>n. A n)) q" |
138 |
proof - |
|
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
139 |
{ |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
140 |
fix s n |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
141 |
have "s \<in> i \<and> v s = n \<longrightarrow> (\<exists>t . Sem (While b c) s t \<and> t \<in> q)" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
142 |
proof (induction "n" arbitrary: s rule: less_induct) |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
143 |
fix n :: nat |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
144 |
fix s :: 'a |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
145 |
assume 1: "\<And>(m::nat) s::'a . m < n \<Longrightarrow> s \<in> i \<and> v s = m \<longrightarrow> (\<exists>t . Sem (While b c) s t \<and> t \<in> q)" |
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
146 |
show "s \<in> i \<and> v s = n \<longrightarrow> (\<exists>t . Sem (While b c) s t \<and> t \<in> q)" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
147 |
proof (rule impI, cases "s \<in> b") |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
148 |
assume 2: "s \<in> b" and "s \<in> i \<and> v s = n" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
149 |
hence "s \<in> i \<inter> b \<inter> {s . v s = n}" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
150 |
using assms(1) by auto |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
151 |
hence "\<exists>t . Sem c s t \<and> t \<in> i \<inter> {s . v s < n}" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
152 |
by (metis assms(2) ValidTC_def) |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
153 |
from this obtain t where 3: "Sem c s t \<and> t \<in> i \<inter> {s . v s < n}" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
154 |
by auto |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
155 |
hence "\<exists>u . Sem (While b c) t u \<and> u \<in> q" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
156 |
using 1 by auto |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
157 |
thus "\<exists>t . Sem (While b c) s t \<and> t \<in> q" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
158 |
using 2 3 Sem.intros(6) by force |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
159 |
next |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
160 |
assume "s \<notin> b" and "s \<in> i \<and> v s = n" |
74503
403ce50e6a2a
separated commands from annotations to be able to abstract about the latter only
nipkow
parents:
72990
diff
changeset
|
161 |
thus "\<exists>t . Sem (While b c) s t \<and> t \<in> q" |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
162 |
using Sem.intros(5) assms(3) by fastforce |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
163 |
qed |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
164 |
qed |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
165 |
} |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
166 |
thus ?thesis |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
167 |
using assms(1) ValidTC_def by force |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
168 |
qed |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
169 |
|
24470
41c81e23c08d
removed Hoare/hoare.ML, Hoare/hoareAbort.ML, ex/svc_oracle.ML (which can be mistaken as attached ML script on case-insensitive file-system);
wenzelm
parents:
21588
diff
changeset
|
170 |
|
72990 | 171 |
subsubsection \<open>Concrete syntax\<close> |
72987
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
172 |
|
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
173 |
setup \<open> |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
174 |
Hoare_Syntax.setup |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
175 |
{Basic = \<^const_syntax>\<open>Basic\<close>, |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
176 |
Skip = \<^const_syntax>\<open>annskip\<close>, |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
177 |
Seq = \<^const_syntax>\<open>Seq\<close>, |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
178 |
Cond = \<^const_syntax>\<open>Cond\<close>, |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
179 |
While = \<^const_syntax>\<open>While\<close>, |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
180 |
Valid = \<^const_syntax>\<open>Valid\<close>, |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
181 |
ValidTC = \<^const_syntax>\<open>ValidTC\<close>} |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
182 |
\<close> |
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
183 |
|
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
184 |
|
72990 | 185 |
subsubsection \<open>Proof methods: VCG\<close> |
72987
b1be35908165
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72985
diff
changeset
|
186 |
|
72985
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
187 |
declare BasicRule [Hoare_Tac.BasicRule] |
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
188 |
and SkipRule [Hoare_Tac.SkipRule] |
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
189 |
and SeqRule [Hoare_Tac.SeqRule] |
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
190 |
and CondRule [Hoare_Tac.CondRule] |
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
191 |
and WhileRule [Hoare_Tac.WhileRule] |
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
192 |
|
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
193 |
declare BasicRuleTC [Hoare_Tac.BasicRuleTC] |
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
194 |
and SkipRuleTC [Hoare_Tac.SkipRuleTC] |
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
195 |
and SeqRuleTC [Hoare_Tac.SeqRuleTC] |
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
196 |
and CondRuleTC [Hoare_Tac.CondRuleTC] |
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
197 |
and WhileRuleTC [Hoare_Tac.WhileRuleTC] |
13682 | 198 |
|
62042 | 199 |
method_setup vcg = \<open> |
72985
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
200 |
Scan.succeed (fn ctxt => SIMPLE_METHOD' (Hoare_Tac.hoare_tac ctxt (K all_tac)))\<close> |
13682 | 201 |
"verification condition generator" |
202 |
||
62042 | 203 |
method_setup vcg_simp = \<open> |
30549 | 204 |
Scan.succeed (fn ctxt => |
72985
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
205 |
SIMPLE_METHOD' (Hoare_Tac.hoare_tac ctxt (asm_full_simp_tac ctxt)))\<close> |
13682 | 206 |
"verification condition generator plus simplification" |
207 |
||
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
208 |
method_setup vcg_tc = \<open> |
72985
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
209 |
Scan.succeed (fn ctxt => SIMPLE_METHOD' (Hoare_Tac.hoare_tc_tac ctxt (K all_tac)))\<close> |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
210 |
"verification condition generator" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
211 |
|
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
212 |
method_setup vcg_tc_simp = \<open> |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
213 |
Scan.succeed (fn ctxt => |
72985
9cc431444435
clarified modules: avoid multiple uses of the same ML file;
wenzelm
parents:
72984
diff
changeset
|
214 |
SIMPLE_METHOD' (Hoare_Tac.hoare_tc_tac ctxt (asm_full_simp_tac ctxt)))\<close> |
72806
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
215 |
"verification condition generator plus simplification" |
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
nipkow
parents:
69605
diff
changeset
|
216 |
|
13682 | 217 |
end |