Minor reformat.
authorballarin
Sun, 31 Oct 2010 11:38:09 +0100
changeset 40293 cd932ab8cb59
parent 40292 ba13793594f0
child 40295 d4923a7f42c1
Minor reformat.
src/HOL/Algebra/Congruence.thy
src/HOL/Algebra/Lattice.thy
--- a/src/HOL/Algebra/Congruence.thy	Sat Oct 30 21:08:20 2010 +0200
+++ b/src/HOL/Algebra/Congruence.thy	Sun Oct 31 11:38:09 2010 +0100
@@ -56,7 +56,8 @@
   fixes S (structure)
   assumes refl [simp, intro]: "x \<in> carrier S \<Longrightarrow> x .= x"
     and sym [sym]: "\<lbrakk> x .= y; x \<in> carrier S; y \<in> carrier S \<rbrakk> \<Longrightarrow> y .= x"
-    and trans [trans]: "\<lbrakk> x .= y; y .= z; x \<in> carrier S; y \<in> carrier S; z \<in> carrier S \<rbrakk> \<Longrightarrow> x .= z"
+    and trans [trans]:
+      "\<lbrakk> x .= y; y .= z; x \<in> carrier S; y \<in> carrier S; z \<in> carrier S \<rbrakk> \<Longrightarrow> x .= z"
 
 (* Lemmas by Stephan Hohe *)
 
--- a/src/HOL/Algebra/Lattice.thy	Sat Oct 30 21:08:20 2010 +0200
+++ b/src/HOL/Algebra/Lattice.thy	Sun Oct 31 11:38:09 2010 +0100
@@ -24,7 +24,8 @@
     and le_trans [trans]:
       "[| x \<sqsubseteq> y; y \<sqsubseteq> z; x \<in> carrier L; y \<in> carrier L; z \<in> carrier L |] ==> x \<sqsubseteq> z"
     and le_cong:
-      "\<lbrakk> x .= y; z .= w; x \<in> carrier L; y \<in> carrier L; z \<in> carrier L; w \<in> carrier L \<rbrakk> \<Longrightarrow> x \<sqsubseteq> z \<longleftrightarrow> y \<sqsubseteq> w"
+      "\<lbrakk> x .= y; z .= w; x \<in> carrier L; y \<in> carrier L; z \<in> carrier L; w \<in> carrier L \<rbrakk> \<Longrightarrow>
+      x \<sqsubseteq> z \<longleftrightarrow> y \<sqsubseteq> w"
 
 definition
   lless :: "[_, 'a, 'a] => bool" (infixl "\<sqsubset>\<index>" 50)