src/HOL/BNF_Greatest_Fixpoint.thy
changeset 69913 ca515cf61651
parent 69605 a96320074298
child 75624 22d1c5f2b9f4
equal deleted inserted replaced
69912:dd55d2c926d9 69913:ca515cf61651
    10 section \<open>Greatest Fixpoint (Codatatype) Operation on Bounded Natural Functors\<close>
    10 section \<open>Greatest Fixpoint (Codatatype) Operation on Bounded Natural Functors\<close>
    11 
    11 
    12 theory BNF_Greatest_Fixpoint
    12 theory BNF_Greatest_Fixpoint
    13 imports BNF_Fixpoint_Base String
    13 imports BNF_Fixpoint_Base String
    14 keywords
    14 keywords
    15   "codatatype" :: thy_decl and
    15   "codatatype" :: thy_defn and
    16   "primcorecursive" :: thy_goal and
    16   "primcorecursive" :: thy_goal_defn and
    17   "primcorec" :: thy_decl
    17   "primcorec" :: thy_defn
    18 begin
    18 begin
    19 
    19 
    20 alias proj = Equiv_Relations.proj
    20 alias proj = Equiv_Relations.proj
    21 
    21 
    22 lemma one_pointE: "\<lbrakk>\<And>x. s = x \<Longrightarrow> P\<rbrakk> \<Longrightarrow> P"
    22 lemma one_pointE: "\<lbrakk>\<And>x. s = x \<Longrightarrow> P\<rbrakk> \<Longrightarrow> P"