tuned whitespace;
authorwenzelm
Mon, 02 Nov 2015 18:30:25 +0100
changeset 61546 53bb4172c7f7
parent 61545 57000ac6291f
child 61547 8494a947fa65
tuned whitespace;
src/HOL/Library/Lattice_Algebras.thy
--- a/src/HOL/Library/Lattice_Algebras.thy	Mon Nov 02 18:09:14 2015 +0100
+++ b/src/HOL/Library/Lattice_Algebras.thy	Mon Nov 02 18:30:25 2015 +0100
@@ -1,4 +1,4 @@
-(* Author: Steven Obua, TU Muenchen *)
+(*  Author:     Steven Obua, TU Muenchen *)
 
 section \<open>Various algebraic structures combined with a lattice\<close>
 
@@ -224,7 +224,7 @@
   proof -
     from that have a: "inf (a + a) 0 = 0"
       by (simp add: inf_commute inf_absorb1)
-    have "inf a 0 + inf a 0 = inf (inf (a + a) 0) a"  (is "?l=_")
+    have "inf a 0 + inf a 0 = inf (inf (a + a) 0) a"  (is "?l = _")
       by (simp add: add_sup_inf_distribs inf_aci)
     then have "?l = 0 + inf a 0"
       by (simp add: a, simp add: inf_commute)
@@ -619,4 +619,3 @@
 qed
 
 end
-