Skip to content

Commit f93e07a

Browse files
committed
fix whitespace, document category solver better
1 parent e73259a commit f93e07a

File tree

2 files changed

+9
-7
lines changed

2 files changed

+9
-7
lines changed

Cubical/Categories/NaturalTransformation/Properties.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -163,9 +163,9 @@ module _ {B : Category ℓB ℓB'}{C : Category ℓC ℓC'}{D : Category ℓD
163163
open Functor
164164
_∘ˡi_ : (K : Functor B C) {G H : Functor C D} (β : NatIso G H)
165165
NatIso (G ∘F K) (H ∘F K)
166-
_∘ˡi_ K β .trans = β .trans ∘ˡ K
166+
_∘ˡi_ K β .trans = β .trans ∘ˡ K
167167
_∘ˡi_ K β .nIso b = β .nIso (K ⟅ b ⟆)
168-
168+
169169
CAT⋆Assoc : {E : Category ℓE ℓE'}
170170
(F : Functor B C)(G : Functor C D)(H : Functor D E)
171171
NatIso (H ∘F (G ∘F F)) ((H ∘F G) ∘F F)

Cubical/Tactics/CategorySolver/Solver.agda

Lines changed: 7 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -24,19 +24,21 @@ module Eval (𝓒 : Category ℓ ℓ') where
2424
𝓘 : Functor FreeCat 𝓟
2525
𝓘 = PseudoYoneda {C = FreeCat}
2626

27-
-- Semantics in 𝓟o 𝓒, interpreting fun symbols using Yoneda
27+
-- Semantics in 𝓟 (𝓒 .ob), interpreting fun symbols using Yoneda
2828
module YoSem = Semantics 𝓟 (𝓘 ∘Interp η)
2929
⟦_⟧yo = YoSem.sem .F-hom
30-
31-
-- | Evaluate by taking the semantics in 𝓟 𝓒 and
32-
-- | use the Yoneda lemma to extract a morphism in 𝓒.
30+
31+
-- | Evaluate by taking the semantics in 𝓟 (𝓒 .ob)
3332
eval : {A B} FreeCat [ A , B ] _
3433
eval {A}{B} e = ⟦ e ⟧yo
3534

35+
-- Evaluation agrees with the Yoneda embedding, and so is fully faithful
3636
Yo-YoSem-agree : 𝓘 ≡ YoSem.sem
3737
Yo-YoSem-agree = YoSem.sem-uniq refl
3838

39-
-- | Eval agrees with the tautological semantics
39+
-- If two expressions in the free category are equal when evaluated
40+
-- in 𝓟 (𝓒 .ob), then they are equal, and so are equal when
41+
-- evaluated in 𝓒.
4042
solve : {A B} (e₁ e₂ : FreeCat [ A , B ])
4143
eval e₁ ≡ eval e₂
4244
⟦ e₁ ⟧c ≡ ⟦ e₂ ⟧c

0 commit comments

Comments
 (0)