Skip to content

Commit

Permalink
feat: port Data.Multiset.Basic change from mathlib3 (leanprover-commu…
Browse files Browse the repository at this point in the history
  • Loading branch information
Ruben-VandeVelde authored and MonadMaverick committed Apr 9, 2023
1 parent 4a951fb commit f9a48d4
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions Mathlib/Data/Multiset/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
! This file was ported from Lean 3 source module data.multiset.basic
! leanprover-community/mathlib commit 2ec920d35348cb2d13ac0e1a2ad9df0fdf1a76b4
! leanprover-community/mathlib commit 06a655b5fcfbda03502f9158bbf6c0f1400886f9
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down Expand Up @@ -3044,9 +3044,9 @@ def Pairwise (r : α → α → Prop) (m : Multiset α) : Prop :=
#align multiset.pairwise Multiset.Pairwise

@[simp]
theorem pairwise_nil (r : α → α → Prop) : Multiset.Pairwise r 0 :=
theorem pairwise_zero (r : α → α → Prop) : Multiset.Pairwise r 0 :=
⟨[], rfl, List.Pairwise.nil⟩
#align multiset.pairwise_nil Multiset.pairwise_nil
#align multiset.pairwise_zero Multiset.pairwise_zero

theorem pairwise_coe_iff {r : α → α → Prop} {l : List α} :
Multiset.Pairwise r l ↔ ∃ l' : List α, l ~ l' ∧ l'.Pairwise r :=
Expand Down

0 comments on commit f9a48d4

Please sign in to comment.