section ‹Q0 abbreviations› theory Q0 imports Set_Theory abbrevs "App" = "❙⋅" and "Abs" = "❙[❙λ_:_. _❙]" and "Eql" = "❙[_ ❙=_❙= _❙]" and "Con" = "❙∧" and "Forall" = "❙[❙∀_:_. _❙]" and "Imp" = "❙⟶" and "Fun" = "❙⇐" begin lemma arg_cong3: "a = b ⟹ c = d ⟹ e = f ⟹ h a c e = h b d f" by auto section ‹Syntax and typing›