Zulip Chat Archive

Stream: maths

Topic: Unfold Multiplication in Group


Charles Murphy (Nov 01 2022 at 01:22):

I am trying to prove that a something is a group and I am wondering if there is a way to get Lean to unfold the definition of multiplication that for the given group.

@[reducible] def C : Type := {n :  // n  -1}

instance : has_mul C :=
{
  mul := λ a b, a.val + b.val + a.val * b.val, sorry⟩,
}

theorem C_mul_one :  a : C, a * 1 = a :=
begin
  intros a,
  cases a,

end

For instance, in the theorem C_mul_one, I get

a_val, a_property * 1 = a_val, a_property

and would like to be able to use the definition of multiplication for C to continue the proof. Thanks.


Last updated: Dec 20 2023 at 11:08 UTC