src/HOL/BNF_Examples/Misc_Primrec.thy
changeset 58231 ad45b22a0b39
parent 55932 68c5104d2204
--- a/src/HOL/BNF_Examples/Misc_Primrec.thy	Mon Sep 08 16:09:10 2014 +0200
+++ b/src/HOL/BNF_Examples/Misc_Primrec.thy	Mon Sep 08 16:14:21 2014 +0200
@@ -35,7 +35,7 @@
   "myrev MyNil = MyNil" |
   "myrev (MyCons x xs) = myapp (myrev xs) (MyCons x MyNil)"
 
-primrec shuffle_sp :: "('a, 'b, 'c, 'd) some_passive \<Rightarrow> ('d, 'a, 'b, 'c) some_passive" where
+primrec shuffle_sp :: "('a \<Colon> ord, 'b \<Colon> ord, 'c, 'd) some_passive \<Rightarrow> ('d, 'a, 'b, 'c) some_passive" where
   "shuffle_sp (SP1 sp) = SP1 (shuffle_sp sp)" |
   "shuffle_sp (SP2 a) = SP3 a" |
   "shuffle_sp (SP3 b) = SP4 b" |