src/HOL/Lattices.thy
changeset 71938 e1b262e7480c
parent 71851 34ecb540a079
child 73411 1f1366966296
--- a/src/HOL/Lattices.thy	Tue Jun 16 08:41:39 2020 +0000
+++ b/src/HOL/Lattices.thy	Tue Jun 16 08:41:39 2020 +0000
@@ -145,16 +145,16 @@
 
 end
 
-text \<open>Passive interpretations for boolean operators\<close>
+text \<open>Interpretations for boolean operators\<close>
 
-lemma semilattice_neutr_and:
-  "semilattice_neutr HOL.conj True"
+interpretation conj: semilattice_neutr \<open>(\<and>)\<close> True
   by standard auto
 
-lemma semilattice_neutr_or:
-  "semilattice_neutr HOL.disj False"
+interpretation disj: semilattice_neutr \<open>(\<or>)\<close> False
   by standard auto
 
+declare conj_assoc [ac_simps del] disj_assoc [ac_simps del] \<comment> \<open>already simp by default\<close>
+
 
 subsection \<open>Syntactic infimum and supremum operations\<close>