tuned orthography
authorhaftmann
Thu, 04 Aug 2011 07:33:08 +0200
changeset 44029 ce4e3090f01a
parent 44028 34abf1f528f3
child 44031 b2158f199652
child 44032 cb768f4ceaf9
tuned orthography
src/HOL/Complete_Lattice.thy
--- a/src/HOL/Complete_Lattice.thy	Thu Aug 04 07:31:59 2011 +0200
+++ b/src/HOL/Complete_Lattice.thy	Thu Aug 04 07:33:08 2011 +0200
@@ -405,7 +405,7 @@
   apply (simp_all add: inf_Sup sup_Inf)*)
 
 subclass distrib_lattice proof -- {* Question: is it sufficient to include @{class distrib_lattice}
-  and proof @{text inf_Sup} and @{text sup_Inf} from that? *}
+  and prove @{text inf_Sup} and @{text sup_Inf} from that? *}
   fix a b c
   from sup_Inf have "a \<squnion> \<Sqinter>{b, c} = (\<Sqinter>d\<in>{b, c}. a \<squnion> d)" .
   then show "a \<squnion> b \<sqinter> c = (a \<squnion> b) \<sqinter> (a \<squnion> c)" by (simp add: INF_def Inf_binary)