src/Doc/Locales/Examples2.thy
changeset 61566 c3d6e570ccef
parent 61419 3c3f8b182e4b
child 67349 0441f2f1b574
--- a/src/Doc/Locales/Examples2.thy	Wed Nov 04 08:13:49 2015 +0100
+++ b/src/Doc/Locales/Examples2.thy	Wed Nov 04 08:13:52 2015 +0100
@@ -2,7 +2,7 @@
 imports Examples
 begin
   interpretation %visible int: partial_order "op \<le> :: [int, int] \<Rightarrow> bool"
-    where "int.less x y = (x < y)"
+    rewrites "int.less x y = (x < y)"
   proof -
     txt \<open>\normalsize The goals are now:
       @{subgoals [display]}