src/HOL/ex/LocaleTest2.thy
changeset 29223 e09c53289830
parent 28823 dcbef866c9e2
child 29226 fcc9606fe141
--- a/src/HOL/ex/LocaleTest2.thy	Wed Dec 10 17:19:25 2008 +0100
+++ b/src/HOL/ex/LocaleTest2.thy	Thu Dec 11 18:30:26 2008 +0100
@@ -433,8 +433,7 @@
 end
 
 
-interpretation dlo < dlat
-(* TODO: definition syntax is unavailable *)
+sublocale dlo < dlat
 proof
   fix x y
   from total have "is_inf x y (if x \<sqsubseteq> y then x else y)" by (auto simp: is_inf_def)
@@ -445,7 +444,7 @@
   then show "EX sup. is_sup x y sup" by blast
 qed
 
-interpretation dlo < ddlat
+sublocale dlo < ddlat
 proof
   fix x y z
   show "x \<sqinter> (y \<squnion> z) = x \<sqinter> y \<squnion> x \<sqinter> z" (is "?l = ?r")