src/HOL/BNF/BNF_LFP.thy
changeset 53305 29c267cb9314
parent 52913 2d2d9d1de1a9
child 53309 42a99f732a40
equal deleted inserted replaced
53304:cfef783090eb 53305:29c267cb9314
     1 (*  Title:      HOL/BNF/BNF_LFP.thy
     1 (*  Title:      HOL/BNF/BNF_LFP.thy
     2     Author:     Dmitriy Traytel, TU Muenchen
     2     Author:     Dmitriy Traytel, TU Muenchen
     3     Copyright   2012
     3     Author:     Lorenz Panny, TU Muenchen
       
     4     Author:     Jasmin Blanchette, TU Muenchen
       
     5     Copyright   2012, 2013
     4 
     6 
     5 Least fixed point operation on bounded natural functors.
     7 Least fixed point operation on bounded natural functors.
     6 *)
     8 *)
     7 
     9 
     8 header {* Least Fixed Point Operation on Bounded Natural Functors *}
    10 header {* Least Fixed Point Operation on Bounded Natural Functors *}
     9 
    11 
    10 theory BNF_LFP
    12 theory BNF_LFP
    11 imports BNF_FP_Basic
    13 imports BNF_FP_Basic
    12 keywords
    14 keywords
    13   "datatype_new" :: thy_decl
    15   "datatype_new" :: thy_decl and
       
    16   "datatype_compat" :: thy_decl
    14 begin
    17 begin
    15 
    18 
    16 lemma subset_emptyI: "(\<And>x. x \<in> A \<Longrightarrow> False) \<Longrightarrow> A \<subseteq> {}"
    19 lemma subset_emptyI: "(\<And>x. x \<in> A \<Longrightarrow> False) \<Longrightarrow> A \<subseteq> {}"
    17 by blast
    20 by blast
    18 
    21 
   230   unfolding vimage2p_def by auto
   233   unfolding vimage2p_def by auto
   231 
   234 
   232 ML_file "Tools/bnf_lfp_util.ML"
   235 ML_file "Tools/bnf_lfp_util.ML"
   233 ML_file "Tools/bnf_lfp_tactics.ML"
   236 ML_file "Tools/bnf_lfp_tactics.ML"
   234 ML_file "Tools/bnf_lfp.ML"
   237 ML_file "Tools/bnf_lfp.ML"
       
   238 ML_file "Tools/bnf_lfp_compat.ML"
   235 
   239 
   236 end
   240 end