src/HOL/HOLCF/IOA/meta_theory/CompoTraces.thy
changeset 48194 1440a3103af0
parent 47239 0b1829860149
child 58318 f95754ca7082
--- a/src/HOL/HOLCF/IOA/meta_theory/CompoTraces.thy	Thu Jul 05 16:11:33 2012 +0200
+++ b/src/HOL/HOLCF/IOA/meta_theory/CompoTraces.thy	Thu Jul 05 16:53:29 2012 +0200
@@ -64,7 +64,10 @@
 axiomatization where
 
 finiteR_mksch:
-  "Finite (mksch A B$tr$x$y) --> Finite tr"
+  "Finite (mksch A B$tr$x$y) \<Longrightarrow> Finite tr"
+
+lemma finiteR_mksch': "\<not> Finite tr \<Longrightarrow> \<not> Finite (mksch A B$tr$x$y)"
+  by (blast intro: finiteR_mksch)
 
 
 declaration {* fn _ => Simplifier.map_ss (Simplifier.set_mksym (K (K NONE))) *}
@@ -507,7 +510,7 @@
 apply (subgoal_tac "schA=UU")
 apply (simp (no_asm_simp))
 (* first side: mksch = UU *)
-apply (auto intro!: ForallQFilterPUU finiteR_mksch [THEN mp, COMP rev_contrapos] ForallBnAmksch)[1]
+apply (auto intro!: ForallQFilterPUU finiteR_mksch' ForallBnAmksch)[1]
 (* schA = UU *)
 apply (erule_tac A = "A" in LastActExtimplUU)
 apply (simp (no_asm_simp))
@@ -726,7 +729,7 @@
 apply (subgoal_tac "schB=UU")
 apply (simp (no_asm_simp))
 (* first side: mksch = UU *)
-apply (force intro!: ForallQFilterPUU finiteR_mksch [THEN mp, COMP rev_contrapos] ForallAnBmksch)
+apply (force intro!: ForallQFilterPUU finiteR_mksch' ForallAnBmksch)
 (* schA = UU *)
 apply (erule_tac A = "B" in LastActExtimplUU)
 apply (simp (no_asm_simp))