Skip to content

Commit

Permalink
chore(data/bool): add bool.lt_iff (#10179)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Nov 5, 2021
1 parent 8991f28 commit 35d3628
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion src/data/bool.lean
Expand Up @@ -173,7 +173,9 @@ instance : linear_order bool :=

@[simp] lemma le_tt {x : bool} : x ≤ tt := or.intro_right _ rfl

@[simp] lemma ff_lt_tt : ff < tt := lt_of_le_of_ne ff_le ff_ne_tt
lemma lt_iff : ∀ {x y : bool}, x < y ↔ x = ff ∧ y = tt := dec_trivial

@[simp] lemma ff_lt_tt : ff < tt := lt_iff.2 ⟨rfl, rfl⟩

lemma le_iff_imp : ∀ {x y : bool}, x ≤ y ↔ (x → y) := dec_trivial

Expand Down

0 comments on commit 35d3628

Please sign in to comment.