Dependent types suck actually

Dependent types suck actually

2025-04-01

STOP DOING DEPENDENT TYPES

Look at what computer scientists have been doing, with all the languages and typecheckers we built for them: (This is REAL dependent types, done by REAL computer scientists)

sq2 : ◀.F-map-iso (◀.F-map-iso (ρ≅ Iso⁻¹)) ∙Iso α≅
    ≡ (α≅ ∙Iso α≅) ∙Iso ▶.F-map-iso (λ≅ Iso⁻¹)
sq2 = ≅-path $
    α→ _ _ _ ∘ ((ρ← ⊗₁ id) ⊗₁ id)    ≡
    (ρ← ⊗₁ ⌜ id ⊗₁ id ⌝) ∘ α→ _ _ _  ≡
    (ρ← ⊗₁ id) ∘ α→ _ _ _            ≡˘
    (id ⊗₁ λ←) ∘ α→ _ _ _ ∘ α→ _ _ _ ∎
theorem integral_re {f : X → 𝕜} (hf : Integrable f μ) :
    ∫ x, RCLike.re (f x) ∂μ = RCLike.re (∫ x, f x ∂μ) :=
  (@RCLike.reCLM 𝕜 _).integral_comp_comm hf
Lemma next_spoke_ring (y : G) : y \in r -> next r y = face (spoke y).
Proof.
move=> ry; have [cycFp Up] := andP ucycFp.
rewrite -{1}[y]nodeK (next_map inj_spoke) ?rev_uniq // (next_rev Up).
rewrite -[prev p _]faceK /spoke ee -(canRL nodeK (nnn y)).
by rewrite (eqP (prev_cycle cycFp _)) // -Ep -Er.
Qed.

"Hello I would like (p : f ∘ g ≡ h ∘ k) apples please"

they have played us for absolute fools





credits