src/HOL/BNF_Composition.thy
changeset 58353 c9f374b64d99
parent 58282 48e16d74845b
child 58889 5b7a9633cfa8
--- a/src/HOL/BNF_Composition.thy	Tue Sep 16 19:23:37 2014 +0200
+++ b/src/HOL/BNF_Composition.thy	Tue Sep 16 19:23:37 2014 +0200
@@ -146,7 +146,8 @@
   rel: "op = :: 'a \<Rightarrow> 'a \<Rightarrow> bool"
   by (auto simp add: Grp_def natLeq_card_order natLeq_cinfinite)
 
-definition id_bnf :: "'a \<Rightarrow> 'a" where "id_bnf \<equiv> (\<lambda>x. x)"
+definition id_bnf :: "'a \<Rightarrow> 'a" where
+  "id_bnf \<equiv> (\<lambda>x. x)"
 
 lemma id_bnf_apply: "id_bnf x = x"
   unfolding id_bnf_def by simp
@@ -177,7 +178,4 @@
   ID.map_id0 ID.map_ident ID.map_transfer ID.rel_Grp ID.rel_compp ID.rel_compp_Grp ID.rel_conversep
   ID.rel_eq ID.rel_flip ID.rel_map ID.rel_mono ID.rel_transfer ID.set_map ID.set_transfer
 
-hide_const (open) id_bnf
-hide_fact (open) id_bnf_def type_definition_id_bnf_UNIV
-
 end