src/HOL/Meson.thy
changeset 61941 31f2105521ee
parent 61799 4cf66f21b764
child 62381 a6479cb85944
--- a/src/HOL/Meson.thy	Sun Dec 27 16:40:09 2015 +0100
+++ b/src/HOL/Meson.thy	Sun Dec 27 17:16:21 2015 +0100
@@ -22,8 +22,7 @@
   and not_exD: "!!P. ~(\<exists>x. P(x)) ==> \<forall>x. ~P(x)"
   by fast+
 
-text \<open>Removal of \<open>-->\<close> and \<open><->\<close> (positive and
-negative occurrences)\<close>
+text \<open>Removal of \<open>\<longrightarrow>\<close> and \<open>\<longleftrightarrow>\<close> (positive and negative occurrences)\<close>
 
 lemma imp_to_disjD: "P-->Q ==> ~P | Q"
   and not_impD: "~(P-->Q) ==> P & ~Q"