src/HOL/HOL.thy
changeset 67443 3abf6a722518
parent 67405 e9ab4ad7bd15
child 67673 c8caefb20564
--- a/src/HOL/HOL.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/HOL.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -1341,8 +1341,7 @@
   if_False
   if_cancel
   if_eq_cancel
-  imp_disjL \<comment>
-   \<open>In general it seems wrong to add distributive laws by default: they
+  imp_disjL \<comment> \<open>In general it seems wrong to add distributive laws by default: they
     might cause exponential blow-up.  But \<open>imp_disjL\<close> has been in for a while
     and cannot be removed without affecting existing proofs.  Moreover,
     rewriting by \<open>(P \<or> Q \<longrightarrow> R) = ((P \<longrightarrow> R) \<and> (Q \<longrightarrow> R))\<close> might be justified on the