src/HOL/BNF_Composition.thy
changeset 67399 eab6ce8368fa
parent 67091 1393c2340eec
child 67613 ce654b0e6d69
equal deleted inserted replaced
67398:5eb932e604a2 67399:eab6ce8368fa
   152 end
   152 end
   153 
   153 
   154 bnf DEADID: 'a
   154 bnf DEADID: 'a
   155   map: "id :: 'a \<Rightarrow> 'a"
   155   map: "id :: 'a \<Rightarrow> 'a"
   156   bd: natLeq
   156   bd: natLeq
   157   rel: "op = :: 'a \<Rightarrow> 'a \<Rightarrow> bool"
   157   rel: "(=) :: 'a \<Rightarrow> 'a \<Rightarrow> bool"
   158   by (auto simp add: natLeq_card_order natLeq_cinfinite)
   158   by (auto simp add: natLeq_card_order natLeq_cinfinite)
   159 
   159 
   160 definition id_bnf :: "'a \<Rightarrow> 'a" where
   160 definition id_bnf :: "'a \<Rightarrow> 'a" where
   161   "id_bnf \<equiv> (\<lambda>x. x)"
   161   "id_bnf \<equiv> (\<lambda>x. x)"
   162 
   162