discontinued presumable workarounds for extra inter-theory space, which are obsolete since 0e5fa27d3293;
authorwenzelm
Tue, 22 Jul 2014 14:52:35 +0200
changeset 57607 5ff0cf3f5f6f
parent 57606 6df377afda4a
child 57608 5d761f9292cf
discontinued presumable workarounds for extra inter-theory space, which are obsolete since 0e5fa27d3293;
src/Doc/Locales/Examples1.thy
src/Doc/Locales/Examples2.thy
src/Doc/Locales/Examples3.thy
--- a/src/Doc/Locales/Examples1.thy	Tue Jul 22 14:36:31 2014 +0200
+++ b/src/Doc/Locales/Examples1.thy	Tue Jul 22 14:52:35 2014 +0200
@@ -1,7 +1,7 @@
 theory Examples1
 imports Examples
 begin
-text {* \vspace{-5ex} *}
+
 section {* Use of Locales in Theories and Proofs
   \label{sec:interpretation} *}
 
--- 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 -
--- a/src/Doc/Locales/Examples3.thy	Tue Jul 22 14:36:31 2014 +0200
+++ b/src/Doc/Locales/Examples3.thy	Tue Jul 22 14:52:35 2014 +0200
@@ -1,7 +1,7 @@
 theory Examples3
 imports Examples
 begin
-text {* \vspace{-5ex} *}
+
 subsection {* Third Version: Local Interpretation
   \label{sec:local-interpretation} *}