Set: pp::colors
  Set: pp::unicode
  Proved: T4
theorem T4 (a b : Bool) (H : a) (H::1 : b) : a ∧ b ∧ a := and_intro H (and_intro H::1 H)