src/Doc/Eisbach/Manual.thy
changeset 67443 3abf6a722518
parent 66453 cc19f7ca2ed6
child 68484 59793df7f853
--- a/src/Doc/Eisbach/Manual.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/Doc/Eisbach/Manual.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -249,16 +249,16 @@
 \<close>
 
     lemmas [intros] =
-      conjI  \<comment>  \<open>@{thm conjI}\<close>
-      impI  \<comment>  \<open>@{thm impI}\<close>
-      disjCI  \<comment>  \<open>@{thm disjCI}\<close>
-      iffI  \<comment>  \<open>@{thm iffI}\<close>
-      notI  \<comment>  \<open>@{thm notI}\<close>
+      conjI  \<comment> \<open>@{thm conjI}\<close>
+      impI  \<comment> \<open>@{thm impI}\<close>
+      disjCI  \<comment> \<open>@{thm disjCI}\<close>
+      iffI  \<comment> \<open>@{thm iffI}\<close>
+      notI  \<comment> \<open>@{thm notI}\<close>
 
     lemmas [elims] =
-      impCE  \<comment>  \<open>@{thm impCE}\<close>
-      conjE  \<comment>  \<open>@{thm conjE}\<close>
-      disjE  \<comment>  \<open>@{thm disjE}\<close>
+      impCE  \<comment> \<open>@{thm impCE}\<close>
+      conjE  \<comment> \<open>@{thm conjE}\<close>
+      disjE  \<comment> \<open>@{thm disjE}\<close>
 
     lemma "(A \<or> B) \<and> (A \<longrightarrow> C) \<and> (B \<longrightarrow> C) \<longrightarrow> C"
       by prop_solver