src/HOL/BNF/BNF_GFP.thy
changeset 52505 e62f3fd2035e
parent 51925 e3b7917186f1
child 52634 7c4b56bac189
equal deleted inserted replaced
52504:52cd8bebc3b6 52505:e62f3fd2035e
   336 by simp
   336 by simp
   337 
   337 
   338 lemma Collect_splitD: "x \<in> Collect (split A) \<Longrightarrow> A (fst x) (snd x)"
   338 lemma Collect_splitD: "x \<in> Collect (split A) \<Longrightarrow> A (fst x) (snd x)"
   339 by auto
   339 by auto
   340 
   340 
   341 lemma spec2: "\<forall>x y. P x y \<Longrightarrow> P x y"
       
   342 by blast
       
   343 
       
   344 ML_file "Tools/bnf_gfp_util.ML"
   341 ML_file "Tools/bnf_gfp_util.ML"
   345 ML_file "Tools/bnf_gfp_tactics.ML"
   342 ML_file "Tools/bnf_gfp_tactics.ML"
   346 ML_file "Tools/bnf_gfp.ML"
   343 ML_file "Tools/bnf_gfp.ML"
   347 
   344 
   348 end
   345 end