src/Doc/Locales/Examples2.thy
changeset 57607 5ff0cf3f5f6f
parent 48985 5386df44a037
child 61419 3c3f8b182e4b
--- a/src/Doc/Locales/Examples2.thy	Tue Jul 22 14:36:31 2014 +0200
+++ b/src/Doc/Locales/Examples2.thy	Tue Jul 22 14:52:35 2014 +0200
@@ -1,7 +1,6 @@
 theory Examples2
 imports Examples
 begin
-text {* \vspace{-5ex} *}
   interpretation %visible int: partial_order "op \<le> :: [int, int] \<Rightarrow> bool"
     where "int.less x y = (x < y)"
   proof -