Skip to content

Commit

Permalink
refactor(topology/local_homeomorph): simpler proof of prod_symm (#5906
Browse files Browse the repository at this point in the history
)

17X smaller proof

co-authors: `lean-gptf`, Stanislas Polu




Co-authored-by: Jesse Michael Han <39395247+jesse-michael-han@users.noreply.github.com>
  • Loading branch information
Jesse Michael Han and jesse-michael-han committed Jan 27, 2021
1 parent a859f10 commit 7244b43
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/topology/local_homeomorph.lean
Expand Up @@ -533,7 +533,7 @@ lemma prod_coe_symm (e : local_homeomorph α β) (e' : local_homeomorph γ δ) :

@[simp, mfld_simps] lemma prod_symm (e : local_homeomorph α β) (e' : local_homeomorph γ δ) :
(e.prod e').symm = (e.symm.prod e'.symm) :=
by ext x; simp [prod_coe_symm]
rfl

@[simp, mfld_simps] lemma prod_trans
{η : Type*} {ε : Type*} [topological_space η] [topological_space ε]
Expand Down

0 comments on commit 7244b43

Please sign in to comment.