Zulip Chat Archive
Stream: general
Topic: simp lemma
Kenny Lau (Sep 07 2018 at 09:40):
Should these two be simp lemmas?
theorem subset_union_left {s₁ s₂ : finset α} : s₁ ⊆ s₁ ∪ s₂ := λ x, mem_union_left _ theorem subset_union_right {s₁ s₂ : finset α} : s₂ ⊆ s₁ ∪ s₂ := λ x, mem_union_right _
Last updated: Dec 20 2023 at 11:08 UTC