Zulip Chat Archive

Stream: lean4

Topic: MIL exercise


Katherine Wei (May 08 2024 at 17:11):

nstance abGrpModule (A : Type) [AddCommGroup₃ A] : Module₁  A where
  smul := zsmul₁
  zero_smul := by exact fun m  rfl
  one_smul := sorry
  mul_smul := sorry
  add_smul := sorry
  smul_add := sorry

I am having problem in these following code. can anyone help me finished the sorry part?

Ted Hwa (May 08 2024 at 19:19):

You can find solutions to all the exercises at https://github.com/leanprover-community/mathematics_in_lean/tree/master/MIL

Within each chapter subdirectory, there is another subdirectory called "solutions". You can consult that whenever you get stuck.


Last updated: May 02 2025 at 03:31 UTC