Skip to content

Commit

Permalink
feat(order/rel_classes): Reflexive relation from irreflexive and vice…
Browse files Browse the repository at this point in the history
…versa (#13411)
  • Loading branch information
vihdzp committed May 26, 2022
1 parent b2973b1 commit 525cc65
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/order/boolean_algebra.lean
Expand Up @@ -812,6 +812,9 @@ instance pi.has_compl {ι : Type u} {α : ι → Type v} [∀ i, has_compl (α i
lemma pi.compl_def {ι : Type u} {α : ι → Type v} [∀ i, has_compl (α i)] (x : Π i, α i) :
xᶜ = λ i, (x i)ᶜ := rfl

instance is_irrefl.compl (r) [is_irrefl α r] : is_refl α rᶜ := ⟨@irrefl α r _⟩
instance is_refl.compl (r) [is_refl α r] : is_irrefl α rᶜ := ⟨λ a, not_not_intro (refl a)⟩

@[simp]
lemma pi.compl_apply {ι : Type u} {α : ι → Type v} [∀ i, has_compl (α i)] (x : Π i, α i) (i : ι) :
xᶜ i = (x i)ᶜ := rfl
Expand Down

0 comments on commit 525cc65

Please sign in to comment.