Closed hrmacbeth closed 3 hours ago
The introduction to the chapter on structures says,
Remember that a non-recursive inductive type that contains only one constructor is called a structure or record.
This appears to need further qualification. Consider the following, which cannot be expressed as a structure:
variable (α β : Type) (f : β → α → α) inductive Foo : α → α → Prop | bar (b : β) (a : α) : Foo a (f b a)
Zulip discussion
Oops, didn't realise this was the Lean 3 repo. Reopened at https://github.com/leanprover/theorem_proving_in_lean4/issues/137.
The introduction to the chapter on structures says,
This appears to need further qualification. Consider the following, which cannot be expressed as a structure:
Zulip discussion