Skip to content

Conversation

@jamesmckinna
Copy link
Contributor

@jamesmckinna jamesmckinna commented Nov 8, 2025

Follows on from #2840 .

Tweaks some of the text introduced there.

@jamesmckinna jamesmckinna added addition status: blocked-by-issue Progress on this issue or PR is blocked by another issue. labels Nov 8, 2025
@jamesmckinna jamesmckinna removed the status: blocked-by-issue Progress on this issue or PR is blocked by another issue. label Nov 11, 2025

∃-≡ : (P : A Set b) {x} P x ↔ (∃[ y ] y ≡ x × P y)
∃-≡ P {x} = mk↔ₛ′ (λ Px x , refl , Px) (λ where (_ , refl , Py) Py)
∃-≡ P {x} = mk↔ₛ′ (⟨ id ⟩⊢⁻ id) (⟨ id ⟩⊢⁺ id)
Copy link
Contributor

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Nice. I wish the proofs could get a similar treatment!

Copy link
Contributor Author

@jamesmckinna jamesmckinna Nov 12, 2025

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Well, ok... but downstream?

I think when I last looked at this, the proofs for the left adjoint behave nicely, while the corresponding ones for the right need (lots of) extensionality, to the point of being unilluminating/incomprehensible.

Also, they should be generalised to
'property of f implies related property of adjoint diagram'
(iso; injective; surjective... adjoint), but I got a headache working out the details...

The special case f = id is almost too special to be worth singling out, but... baby steps. It's one reason I went back on my original thought to rewrite the lemma statement to use the adjoint notation... it felt like overkill for too-small stakes.

Copy link
Contributor Author

@jamesmckinna jamesmckinna Nov 12, 2025

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Oh, and the use of id to proxy for its definitionally-equal ⊆-refl (Yoneda lemma!) is a bit cheeky, but arguably it looks worse by using the (conceptually) type-correct version, cf. the functoriality proofs, which I wrote Yoneda-style, rather than flattening out the compositions to re duplicate the pattern-matching versions which precede them...

Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

Projects

None yet

Development

Successfully merging this pull request may close these issues.

2 participants