Skip to content

Commit

Permalink
chore: add doc explanations
Browse files Browse the repository at this point in the history
  • Loading branch information
fgdorais committed Oct 27, 2023
1 parent 85ba850 commit a3484a1
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions Std/Data/Bool.lean
Original file line number Diff line number Diff line change
Expand Up @@ -76,6 +76,7 @@ theorem and_eq_true_iff : ∀ (x y : Bool), (x && y) = true ↔ x = true ∧ y =
theorem and_eq_false_iff : ∀ (x y : Bool), (x && y) = false ↔ x = false ∨ y = false := by
decide

/-! non infix aliases -/
alias and_not_self_left := Bool.not_and_self
alias and_not_self_right := Bool.and_not_self
alias and_false_left := Bool.false_and
Expand Down Expand Up @@ -116,6 +117,7 @@ theorem or_eq_true_iff : ∀ (x y : Bool), (x || y) = true ↔ x = true ∨ y =
theorem or_eq_false_iff : ∀ (x y : Bool), (x || y) = false ↔ x = false ∧ y = false := by
decide

/-! non infix aliases -/
alias or_not_self_left := Bool.not_or_self
alias or_not_self_right := Bool.or_not_self
alias or_false_left := Bool.false_or
Expand Down Expand Up @@ -168,6 +170,7 @@ theorem xor_right_comm : ∀ (x y z : Bool), xor (xor x y) z = xor (xor x z) y :
theorem xor_assoc : ∀ (x y z : Bool), xor (xor x y) z = xor x (xor y z) := by
decide

/-! non infix aliases -/
alias xor_not_self_left := Bool.not_xor_self
alias xor_not_self_right := Bool.xor_not_self
alias xor_not_left := Bool.not_xor
Expand Down

0 comments on commit a3484a1

Please sign in to comment.