tuned;
authorwenzelm
Fri, 06 Oct 2000 01:21:17 +0200
changeset 10158 00fdd5c330ea
parent 10157 6d3987f3aad9
child 10159 a72ddfdbfca0
tuned;
src/HOL/Lattice/Lattice.thy
--- a/src/HOL/Lattice/Lattice.thy	Fri Oct 06 01:04:56 2000 +0200
+++ b/src/HOL/Lattice/Lattice.thy	Fri Oct 06 01:21:17 2000 +0200
@@ -384,7 +384,7 @@
 
 text {*
   The class of lattices is closed under direct binary products (cf.\
-  also \S\ref{sec:prod-order}).
+  \S\ref{sec:prod-order}).
 *}
 
 lemma is_inf_prod: "is_inf p q (fst p \<sqinter> fst q, snd p \<sqinter> snd q)"
@@ -472,7 +472,7 @@
 
 text {*
   The class of lattices is closed under general products (function
-  spaces) as well (cf.\ also \S\ref{sec:fun-order}).
+  spaces) as well (cf.\ \S\ref{sec:fun-order}).
 *}
 
 lemma is_inf_fun: "is_inf f g (\<lambda>x. f x \<sqinter> g x)"