avoid dependence on adm_tac solver
authorhuffman
Mon, 22 Mar 2010 15:42:07 -0700
changeset 35907 ea0bf2a01eb0
parent 35906 e0382e4b4da7
child 35908 21e45c81e828
avoid dependence on adm_tac solver
src/HOLCF/IOA/meta_theory/Sequence.thy
--- a/src/HOLCF/IOA/meta_theory/Sequence.thy	Mon Mar 22 15:23:16 2010 -0700
+++ b/src/HOLCF/IOA/meta_theory/Sequence.thy	Mon Mar 22 15:42:07 2010 -0700
@@ -814,9 +814,8 @@
 
 lemma nForall_HDFilter:
  "~Forall P y --> (? x. HD$(Filter (%a. ~P a)$y) = Def x)"
-(* Pay attention: is only admissible with chain-finite package to be added to
-        adm test *)
-apply (rule_tac x="y" in Seq_induct)
+unfolding not_Undef_is_Def [symmetric]
+apply (induct y rule: Seq_induct)
 apply (simp add: Forall_def sforall_def)
 apply simp_all
 done