Skip to content

Commit

Permalink
forgor
Browse files Browse the repository at this point in the history
  • Loading branch information
Bergschaf committed Jan 3, 2025
1 parent df93506 commit fe4ddc1
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Order/CompleteBooleanAlgebra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -490,7 +490,7 @@ theorem sdiff_eq_sInf : a \ b = sInf {w | a ≤ b ⊔ w} :=
(isLeast_sdiff a b).isGLB.sInf_eq.symm

theorem hnot_eq_sInf_codisjoint : ¬a = sInf {w | Codisjoint a w} := by
simp_rw [← Coframe.top_sdiff,sdiff_eq_sInf,codisjoint_iff]
simp [← Coframe.top_sdiff,sdiff_eq_sInf,codisjoint_iff,sup_comm]

-- see Note [lower instance priority]
instance (priority := 100) Coframe.toDistribLattice : DistribLattice α where
Expand Down

0 comments on commit fe4ddc1

Please sign in to comment.