src/LCF/ex/Ex3.thy
changeset 58977 9576b510f6a2
parent 58974 cbc2ac19d783
child 60770 240563fbf41d
--- a/src/LCF/ex/Ex3.thy	Tue Nov 11 13:50:56 2014 +0100
+++ b/src/LCF/ex/Ex3.thy	Tue Nov 11 15:55:31 2014 +0100
@@ -5,8 +5,8 @@
 begin
 
 axiomatization
-  s     :: "'a => 'a" and
-  p     :: "'a => 'a => 'a"
+  s     :: "'a \<Rightarrow> 'a" and
+  p     :: "'a \<Rightarrow> 'a \<Rightarrow> 'a"
 where
   p_strict:     "p(UU) = UU" and
   p_s:          "p(s(x),y) = s(p(x,y))"