removed unnecessary lemmas
authornipkow
Mon, 02 Jan 2012 11:33:50 +0100
changeset 46069 4869f1389333
parent 46068 b9d4ec0f79ac
child 46070 8392c28d7868
removed unnecessary lemmas
src/HOL/IMP/Collecting.thy
--- a/src/HOL/IMP/Collecting.thy	Mon Jan 02 10:51:28 2012 +0100
+++ b/src/HOL/IMP/Collecting.thy	Mon Jan 02 11:33:50 2012 +0100
@@ -136,27 +136,6 @@
 lemma le_post: "c \<le> d \<Longrightarrow> post c \<le> post d"
 by(induction c d rule: less_eq_acom.induct) auto
 
-lemma le_strip: "c \<le> d \<Longrightarrow> strip c = strip d"
-by(induction c d rule: less_eq_acom.induct) auto
-
-lemma le_SKIP_iff: "c \<le> SKIP {P'} \<longleftrightarrow> (EX P. c = SKIP {P} \<and> P \<le> P')"
-by (cases c) simp_all
-
-lemma le_Assign_iff: "c \<le> x::=e {P'} \<longleftrightarrow> (EX P. c = x::=e {P} \<and> P \<le> P')"
-by (cases c) simp_all
-
-lemma le_Semi_iff: "c \<le> d1;d2 \<longleftrightarrow> (EX c1 c2. c = c1;c2 \<and> c1 \<le> d1 \<and> c2 \<le> d2)"
-by (cases c) simp_all
-
-lemma le_If_iff: "c \<le> IF b THEN d1 ELSE d2 {P'} \<longleftrightarrow>
-  (EX c1 c2 P. c = IF b THEN c1 ELSE c2 {P} \<and> c1 \<le> d1 \<and> c2 \<le> d2 \<and> P \<le> P')"
-by (cases c) simp_all
-
-lemma le_While_iff: "c \<le> {I'} WHILE b DO d {P'} \<longleftrightarrow>
-  (EX I c' P. c = {I} WHILE b DO c' {P} \<and> I \<le> I' \<and> c' \<le> d \<and> P \<le> P')"
-by (cases c) auto
-
-
 subsubsection "Collecting semantics"
 
 fun step :: "state set \<Rightarrow> state set acom \<Rightarrow> state set acom" where