src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy
changeset 61169 4de9ff3ea29a
parent 58889 5b7a9633cfa8
child 61942 f02b26f7d39d
--- a/src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy	Sun Sep 13 22:25:21 2015 +0200
+++ b/src/HOL/Quickcheck_Examples/Quickcheck_Examples.thy	Sun Sep 13 22:56:52 2015 +0200
@@ -478,8 +478,8 @@
   fixes R
   assumes "R x y --> R y x --> x = y"
 
-interpretation equal : antisym "op =" by default simp
-interpretation order_nat : antisym "op <= :: nat => _ => _" by default simp
+interpretation equal : antisym "op =" by standard simp
+interpretation order_nat : antisym "op <= :: nat => _ => _" by standard simp
 
 lemma (in antisym)
   "R x y --> R y z --> R x z"