src/HOL/BNF/BNF_LFP.thy
changeset 52731 dacd47a0633f
parent 52635 4f84b730c489
child 52913 2d2d9d1de1a9
equal deleted inserted replaced
52730:6bf02eb4ddf7 52731:dacd47a0633f
   224 lemma meta_spec2:
   224 lemma meta_spec2:
   225   assumes "(\<And>x y. PROP P x y)"
   225   assumes "(\<And>x y. PROP P x y)"
   226   shows "PROP P x y"
   226   shows "PROP P x y"
   227 by (rule `(\<And>x y. PROP P x y)`)
   227 by (rule `(\<And>x y. PROP P x y)`)
   228 
   228 
       
   229 lemma vimage2p_fun_rel: "(fun_rel (vimage2p f g R) R) f g"
       
   230   unfolding fun_rel_def vimage2p_def by auto
       
   231 
       
   232 lemma predicate2D_vimage2p: "\<lbrakk>R \<le> vimage2p f g S; R x y\<rbrakk> \<Longrightarrow> S (f x) (g y)"
       
   233   unfolding vimage2p_def by auto
       
   234 
   229 ML_file "Tools/bnf_lfp_util.ML"
   235 ML_file "Tools/bnf_lfp_util.ML"
   230 ML_file "Tools/bnf_lfp_tactics.ML"
   236 ML_file "Tools/bnf_lfp_tactics.ML"
   231 ML_file "Tools/bnf_lfp.ML"
   237 ML_file "Tools/bnf_lfp.ML"
   232 
   238 
   233 end
   239 end