Skip to content

Commit 420374b

Browse files
committed
missing lemma
1 parent a4b0cef commit 420374b

File tree

2 files changed

+15
-12
lines changed

2 files changed

+15
-12
lines changed

FLT/for_mathlib/Coalgebra/Monoid.lean

+12
Original file line numberDiff line numberDiff line change
@@ -203,4 +203,16 @@ lemma mul_repr {ι : Type* } (a : A) (ℐ : Finset ι) (Δ₁ Δ₂ : ι → A)
203203

204204
attribute [deprecated] mul_assoc' mul_one' one_mul'
205205

206+
section commutative_bialgebra
207+
208+
variable {A' : Type*} [CommSemiring A'] [Bialgebra R A']
209+
210+
lemma comp_one {A' : Type*} [CommSemiring A'] [Bialgebra R A']
211+
(f : AlgHomPoint R A' L) :
212+
f.comp (1 : AlgHomPoint R A' A') = 1 := by
213+
ext
214+
simp [one_def, Algebra.ofId_apply, Algebra.algebraMap_eq_smul_one, f.map_smul, f.map_one]
215+
216+
end commutative_bialgebra
217+
206218
end AlgHomPoint

FLT/for_mathlib/HopfAlgebra/Basic.lean

+3-12
Original file line numberDiff line numberDiff line change
@@ -148,25 +148,16 @@ noncomputable instance instGroup : Group (AlgHomPoint R A L) where
148148
end AlgHomPoint
149149

150150
lemma antipodeAlgHom_inv : antipodeAlgHom⁻¹ = AlgHom.id R A :=
151-
inv_eq_iff_mul_eq_one.mpr <| AlgHom.ext fun x ↦ congr($(antipode_mul_id) x)
151+
inv_eq_iff_mul_eq_one.mpr <| mul_eq_one_iff_eq_inv.mpr rfl
152152

153153
lemma antipodeAlgHom_mul_id : antipodeAlgHom * AlgHom.id R A = 1 :=
154154
AlgHom.ext fun _ ↦ congr($(antipode_mul_id) _)
155155

156-
157156
lemma id_mul_antipodeAlgHom : AlgHom.id R A * antipodeAlgHom = 1 :=
158157
AlgHom.ext fun _ ↦ congr($(id_mul_antipode) _)
159158

160-
lemma antipodeAlgHom_square : antipodeAlgHom.comp antipodeAlgHom = AlgHom.id R A := by
161-
suffices antipodeAlgHom * (antipodeAlgHom.comp antipodeAlgHom) = (1 : AlgHomPoint R A A) by
162-
conv_rhs at this => rw [← antipodeAlgHom_mul_id]
163-
simpa only [mul_right_inj] using this
164-
ext a
165-
simp_rw [AlgHomPoint.mul_repr (repr := Coalgebra.comul_repr a),
166-
AlgHom.coe_comp, Function.comp_apply, ← antipodeAlgHom.map_mul, ← map_sum,
167-
antipodeAlgHom_apply, antipode_repr_eq_smul' (repr := Coalgebra.comul_repr a), map_smul,
168-
antipode_one, Algebra.smul_def, mul_one]
169-
rfl
159+
lemma antipodeAlgHom_square : antipodeAlgHom.comp antipodeAlgHom = AlgHom.id R A :=
160+
antipodeAlgHom_inv
170161

171162
/--
172163
Then antipode map is an algebra equivalence.

0 commit comments

Comments
 (0)