Commit 2022-11-07 03:12 99667781
View on Github →feat: port data.bool.basic (#534) Issues that came up:
- my understanding of the lean 4 naming convention is that capital/small letter choices are often dictated to you. However Lean 4 has notfor bools andNotfor props. This causes the following issue: in my port I have gone for the name
 What should this theorem be called? The algorithm saystheorem Not_eq_not : ∀ {a b : Bool}, ¬a = !b ↔ a = bnot_eq_notwhich is misleading...or is it? It comes up a few times (the others arenot_iff_NotandNot_not_eq)
- When defining LinearOrder I had to do a lot of unfolding which is not present in Lean 3.
instance : LinearOrder Bool where
  le := fun a b => a = false ∨ b = true
  le_refl := by unfold LE.le; decide
  le_trans := by unfold LE.le; decide
  le_antisymm := by unfold LE.le Preorder.toLE; decide
  le_total := by unfold LE.le Preorder.toLE PartialOrder.toPreorder; decide
  decidable_le := by unfold LE.le Preorder.toLE PartialOrder.toPreorder; exact inferInstance
...
- Again on orders: lt_iff_le_not_leis not an autoparam so I had to prove it explicitly withIff.rfl. Do autoparams exist in Lean 4 yet? Does this need to be flagged?
- Because the names of many functions on booleans changed (bor->or,bnot->notetc) I had to #align a lot of stuff. However the namespace also changed (bool->Bool). Am I right in thinking that the few theorems likebool.lt_iff, which becomesBool.lt_iff(i.e. the theorem name itself survived the naming change but the namespace did not) do not need to be #align ed?