src/HOL/BNF_LFP.thy
changeset 55534 b18bdcbda41b
parent 55531 601ca8efa000
child 55538 6a5986170c1d
equal deleted inserted replaced
55533:6260caf1d612 55534:b18bdcbda41b
    11 
    11 
    12 theory BNF_LFP
    12 theory BNF_LFP
    13 imports BNF_FP_Base
    13 imports BNF_FP_Base
    14 keywords
    14 keywords
    15   "datatype_new" :: thy_decl and
    15   "datatype_new" :: thy_decl and
    16   "datatype_compat" :: thy_decl
    16   "datatype_compat" :: thy_decl and
       
    17   "primrec" :: thy_decl
    17 begin
    18 begin
    18 
    19 
    19 lemma subset_emptyI: "(\<And>x. x \<in> A \<Longrightarrow> False) \<Longrightarrow> A \<subseteq> {}"
    20 lemma subset_emptyI: "(\<And>x. x \<in> A \<Longrightarrow> False) \<Longrightarrow> A \<subseteq> {}"
    20 by blast
    21 by blast
    21 
    22