# HG changeset patch # User haftmann # Date 1312435988 -7200 # Node ID ce4e3090f01a9742010182508d3e6963be5bc6f1 # Parent 34abf1f528f39eb0603302bbbe392e0dbf143c9a tuned orthography diff -r 34abf1f528f3 -r ce4e3090f01a 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 \ \{b, c} = (\d\{b, c}. a \ d)" . then show "a \ b \ c = (a \ b) \ (a \ c)" by (simp add: INF_def Inf_binary)