swap False to the right in assumptions to be eliminated at the right end
authornipkow
Sun, 03 May 2015 15:38:25 +0200
changeset 60169 5ef8ed685965
parent 60168 0305c511a821
child 60170 031ec3d34d31
swap False to the right in assumptions to be eliminated at the right end
src/HOL/Extraction.thy
src/HOL/HOL.thy
src/HOL/Hoare_Parallel/OG_Examples.thy
--- a/src/HOL/Extraction.thy	Fri May 01 20:26:06 2015 +0200
+++ b/src/HOL/Extraction.thy	Sun May 03 15:38:25 2015 +0200
@@ -32,7 +32,7 @@
   induct_atomize induct_atomize' induct_rulify induct_rulify'
   induct_rulify_fallback induct_trueI
   True_implies_equals implies_True_equals TrueE
-  False_implies_equals
+  False_implies_equals implies_False_swap
 
 lemmas [extraction_expand_def] =
   HOL.induct_forall_def HOL.induct_implies_def HOL.induct_equal_def HOL.induct_conj_def
--- a/src/HOL/HOL.thy	Fri May 01 20:26:06 2015 +0200
+++ b/src/HOL/HOL.thy	Sun May 03 15:38:25 2015 +0200
@@ -1270,6 +1270,10 @@
 lemma False_implies_equals: "(False \<Longrightarrow> P) \<equiv> Trueprop True"
 by default simp_all
 
+lemma implies_False_swap: "NO_MATCH (Trueprop False) P \<Longrightarrow>
+  (False \<Longrightarrow> PROP P \<Longrightarrow> PROP Q) \<equiv> (PROP P \<Longrightarrow> False \<Longrightarrow> PROP Q)"
+by(rule swap_prems_eq)
+
 lemma ex_simps:
   "!!P Q. (EX x. P x & Q)   = ((EX x. P x) & Q)"
   "!!P Q. (EX x. P & Q x)   = (P & (EX x. Q x))"
@@ -1293,7 +1297,7 @@
 lemmas [simp] =
   triv_forall_equality (*prunes params*)
   True_implies_equals implies_True_equals (*prune True in asms*)
-  False_implies_equals (*prune False in asms*)
+  False_implies_equals implies_False_swap (*prune False in asms*)
   if_True
   if_False
   if_cancel
--- a/src/HOL/Hoare_Parallel/OG_Examples.thy	Fri May 01 20:26:06 2015 +0200
+++ b/src/HOL/Hoare_Parallel/OG_Examples.thy	Sun May 03 15:38:25 2015 +0200
@@ -191,7 +191,7 @@
 apply force
 --\<open>6 subgoals left\<close>
 prefer 6
-apply(erule_tac x=i in allE)
+apply(erule_tac x=j in allE)
 apply fastforce
 --\<open>5 subgoals left\<close>
 prefer 5