doc-src/Locales/Locales/Examples.thy
changeset 29293 d4ef21262b8f
parent 27375 8d2c3d61c502
child 29567 286c01be90cb
--- a/doc-src/Locales/Locales/Examples.thy	Thu Jan 01 20:28:03 2009 +0100
+++ b/doc-src/Locales/Locales/Examples.thy	Thu Jan 01 20:56:23 2009 +0100
@@ -610,7 +610,7 @@
   Changes to the locale hierarchy may be declared
   with the \isakeyword{interpretation} command. *}
 
-  interpretation %visible total_order \<subseteq> lattice
+  sublocale %visible total_order \<subseteq> lattice
 
 txt {* This enters the context of locale @{text total_order}, in
   which the goal @{subgoals [display]} must be shown.  First, the
@@ -652,7 +652,7 @@
 
 text {* Similarly, total orders are distributive lattices. *}
 
-  interpretation total_order \<subseteq> distrib_lattice
+  sublocale total_order \<subseteq> distrib_lattice
   proof unfold_locales
     fix %"proof" x y z
     show "x \<sqinter> (y \<squnion> z) = x \<sqinter> y \<squnion> x \<sqinter> z" (is "?l = ?r")