generalized type signature to permit overloading on `set`
authorhaftmann
Sat, 24 Dec 2011 15:53:09 +0100
changeset 45965 2af982715e5c
parent 45964 7b3a18670a9f
child 45966 03ce2b2a29a2
generalized type signature to permit overloading on `set`
src/HOL/Nat.thy
--- a/src/HOL/Nat.thy	Sat Dec 24 15:53:08 2011 +0100
+++ b/src/HOL/Nat.thy	Sat Dec 24 15:53:09 2011 +0100
@@ -1200,9 +1200,9 @@
   functions and relations, in order to share the same syntax.
 *}
 
-consts compow :: "nat \<Rightarrow> ('a \<Rightarrow> 'b) \<Rightarrow> ('a \<Rightarrow> 'b)"
+consts compow :: "nat \<Rightarrow> 'a \<Rightarrow> 'a"
 
-abbreviation compower :: "('a \<Rightarrow> 'b) \<Rightarrow> nat \<Rightarrow> 'a \<Rightarrow> 'b" (infixr "^^" 80) where
+abbreviation compower :: "'a \<Rightarrow> nat \<Rightarrow> 'a" (infixr "^^" 80) where
   "f ^^ n \<equiv> compow n f"
 
 notation (latex output)