src/HOL/BNF_GFP.thy
changeset 55538 6a5986170c1d
parent 55463 942c2153b5b4
child 55542 4394bb0b522b
equal deleted inserted replaced
55537:6ec3c2c38650 55538:6a5986170c1d
   347   then obtain x where x: "x \<in> A" and X: "X = proj r x" using ECH proj_image[of r A] by blast
   347   then obtain x where x: "x \<in> A" and X: "X = proj r x" using ECH proj_image[of r A] by blast
   348   hence "univ f X = f x" using assms univ_commute by fastforce
   348   hence "univ f X = f x" using assms univ_commute by fastforce
   349   thus "univ f X \<in> B" using x PRES by simp
   349   thus "univ f X \<in> B" using x PRES by simp
   350 qed
   350 qed
   351 
   351 
   352 ML_file "Tools/BNF/bnf_gfp_rec_sugar_tactics.ML"
       
   353 ML_file "Tools/BNF/bnf_gfp_rec_sugar.ML"
       
   354 ML_file "Tools/BNF/bnf_gfp_util.ML"
   352 ML_file "Tools/BNF/bnf_gfp_util.ML"
   355 ML_file "Tools/BNF/bnf_gfp_tactics.ML"
   353 ML_file "Tools/BNF/bnf_gfp_tactics.ML"
   356 ML_file "Tools/BNF/bnf_gfp.ML"
   354 ML_file "Tools/BNF/bnf_gfp.ML"
       
   355 ML_file "Tools/BNF/bnf_gfp_rec_sugar_tactics.ML"
       
   356 ML_file "Tools/BNF/bnf_gfp_rec_sugar.ML"
   357 
   357 
   358 end
   358 end