Skip to content

Commit

Permalink
feat(logic/function/basic): a lemma on symmetric operations and flip (#…
Browse files Browse the repository at this point in the history
…7871)

This lemma is used to show that if multiplication is commutative, then `flip`ping the arguments returns the same function.

This is used in PR #7645 .

Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
  • Loading branch information
adomani and eric-wieser committed Jun 10, 2021
1 parent f2a0897 commit ba00a23
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/logic/function/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -654,3 +654,6 @@ lemma cast_inj {α β : Type*} (h : α = β) {x y : α} : cast h x = cast h y
if for each pair of distinct points there is a function taking different values on them. -/
def set.separates_points {α β : Type*} (A : set (α → β)) : Prop :=
∀ ⦃x y : α⦄, x ≠ y → ∃ f ∈ A, (f x : β) ≠ f y

lemma is_symm_op.flip_eq {α β} (op) [is_symm_op α β op] : flip op = op :=
funext $ λ a, funext $ λ b, (is_symm_op.symm_op a b).symm

0 comments on commit ba00a23

Please sign in to comment.