Zulip Chat Archive
Stream: mathlib4
Topic: spelling of assumption set being the complement
Christian Merten (Dec 04 2024 at 11:37):
Which of these is the preferred spelling for assuming that two sets s and t are each others complement?
import Mathlib.Data.Set.Basic
variable {α : Type} {s t : Set α}
lemma opt1 (h : IsCompl s t) : True := trivial
lemma opt2 (h₁ : s ∪ t = Set.univ) (h₂ : s ∩ t = ∅) : True := trivial
lemma opt3 (h : s = tᶜ) : True := trivial
(All of these are in simp normal form).
Yaël Dillies (Dec 04 2024 at 11:40):
The first one
Christian Merten (Dec 04 2024 at 11:40):
Thanks
Yaël Dillies (Dec 04 2024 at 11:40):
But usually you would write s and s^compl. Is there a reason you are not doing that?
Christian Merten (Dec 04 2024 at 11:43):
Yes, the precise setup is I have two (injective) functions α → β and γ → β and I want to define a basis indexed by γ under the assumption that the images are complements in β.
Last updated: May 02 2025 at 03:31 UTC