Skip to content

Commit a02b532

Browse files
committed
chore: golf using funext₂ (#21106)
1 parent 77d9317 commit a02b532

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/Order/Antisymmetrization.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -40,7 +40,7 @@ def AntisymmRel (a b : α) : Prop :=
4040
r a b ∧ r b a
4141

4242
theorem antisymmRel_swap : AntisymmRel (swap r) = AntisymmRel r :=
43-
funext fun _ => funext fun _ => propext and_comm
43+
funext fun _ _ ↦ propext and_comm
4444

4545
@[refl]
4646
theorem antisymmRel_refl [IsRefl α r] (a : α) : AntisymmRel r a a :=

0 commit comments

Comments
 (0)