src/HOLCF/Cfun.thy
changeset 25135 4f8176c940cf
parent 25131 2c8caac48ade
child 25701 73fbe868b4e7
--- a/src/HOLCF/Cfun.thy	Sun Oct 21 14:53:44 2007 +0200
+++ b/src/HOLCF/Cfun.thy	Sun Oct 21 16:27:42 2007 +0200
@@ -435,18 +435,18 @@
 
 subsection {* Identity and composition *}
 
-consts
-  ID      :: "'a \<rightarrow> 'a"
-  cfcomp  :: "('b \<rightarrow> 'c) \<rightarrow> ('a \<rightarrow> 'b) \<rightarrow> 'a \<rightarrow> 'c"
+definition
+  ID :: "'a \<rightarrow> 'a" where
+  "ID = (\<Lambda> x. x)"
+
+definition
+  cfcomp  :: "('b \<rightarrow> 'c) \<rightarrow> ('a \<rightarrow> 'b) \<rightarrow> 'a \<rightarrow> 'c" where
+  oo_def: "cfcomp = (\<Lambda> f g x. f\<cdot>(g\<cdot>x))"
 
 abbreviation
   cfcomp_syn :: "['b \<rightarrow> 'c, 'a \<rightarrow> 'b] \<Rightarrow> 'a \<rightarrow> 'c"  (infixr "oo" 100)  where
   "f oo g == cfcomp\<cdot>f\<cdot>g"
 
-defs
-  ID_def: "ID \<equiv> (\<Lambda> x. x)"
-  oo_def: "cfcomp \<equiv> (\<Lambda> f g x. f\<cdot>(g\<cdot>x))" 
-
 lemma ID1 [simp]: "ID\<cdot>x = x"
 by (simp add: ID_def)