diff -r 61e4c96bf2b6 -r ad45b22a0b39 src/HOL/BNF_Examples/Misc_Primrec.thy --- 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 \ ('d, 'a, 'b, 'c) some_passive" where +primrec shuffle_sp :: "('a \ ord, 'b \ ord, 'c, 'd) some_passive \ ('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" |