]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/ground/lib/bool_and.ma
update in delayed_updating and ground
[helm.git] / matita / matita / contribs / lambdadelta / ground / lib / bool_and.ma
index b7a8bf96422c190db6ea808b4ba9342632ba0f67..680ead78718faf9754e0c300989c8ddcb6088a1d 100644 (file)
@@ -23,16 +23,27 @@ lemma commutative_andb:
 * * // qed.
 
 lemma andb_false_dx (b):
-      (b ∧ Ⓕ) = Ⓕ.
+      Ⓕ = (b ∧ Ⓕ).
 * // qed.
 
 lemma andb_false_sn (b):
-      (Ⓕ ∧ b) = Ⓕ.
+      Ⓕ = (Ⓕ ∧ b).
+// qed.
+
+lemma andb_true_dx (b):
+      b = (b ∧ Ⓣ).
+* // qed.
+
+lemma andb_true_sn (b):
+      b = (Ⓣ ∧ b).
 // qed.
 
 (* Advanced inversions ******************************************************)
 
-lemma andb_inv_true_dx (b1) (b2):
-      (b1 ∧ b2) = Ⓣ → ∧∧ b1 = Ⓣ & b2 = Ⓣ.
-* normalize /2 width=1 by conj/ #b2 #H destruct
+lemma andb_inv_true_sn (b1) (b2):
+      Ⓣ = (b1 ∧ b2) → ∧∧ Ⓣ = b1 & Ⓣ = b2.
+* normalize
+[ /2 width=1 by conj/
+| #b2 #H destruct
+]
 qed-.