formal passive interpretation proofs for conj and disj
authorhaftmann
Wed, 10 Aug 2016 18:57:20 +0200
changeset 63661 92e037803666
parent 63660 76302202a92d
child 63662 5cdcd51a4dad
formal passive interpretation proofs for conj and disj
src/HOL/Lattices.thy
--- a/src/HOL/Lattices.thy	Mon Aug 08 14:01:49 2016 +0200
+++ b/src/HOL/Lattices.thy	Wed Aug 10 18:57:20 2016 +0200
@@ -139,6 +139,16 @@
 
 end
 
+text \<open>Passive interpretations for boolean operators\<close>
+
+lemma semilattice_neutr_and:
+  "semilattice_neutr HOL.conj True"
+  by standard auto
+
+lemma semilattice_neutr_or:
+  "semilattice_neutr HOL.disj False"
+  by standard auto
+
 
 subsection \<open>Syntactic infimum and supremum operations\<close>