Commit graph

10 commits

Author SHA1 Message Date
Frederik Hanghøj Iversen 360e2b95dd Make parameter to monad equivalence explicit 2018-03-14 11:20:07 +01:00
Frederik Hanghøj Iversen 7aec22b30a Expose both monad formulations qualified from Cat.Category.Monad 2018-03-14 11:00:52 +01:00
Frederik Hanghøj Iversen 6229decfb2 Merge branch 'master' into dev 2018-03-14 10:50:57 +01:00
Frederik Hanghøj Iversen 41e2d02c8d [WIP] Prove voe §2.3
By Andrea

The reason you cannot use cong in [1] is that §2-fromMonad result type
depends on the input, you need a dependent version of cong:

cong-d : ∀ {ℓ} {A : Set ℓ} {ℓ'} {B : A → Set ℓ'} {x y : A}
               → (f : (x : A) → B x)
               → (eq : x ≡ y)
               → PathP (\ i → B (eq i)) (f x) (f y)
cong-d f p = λ i → f (p i)

I attach a modified Voevodsky.agda.

Notice that the definition of "t" is still highlighted in yellow,
that's because it being a homogeneous path depends on the exact
definition of lem, see the comment with the two definitional equality
constraints.
2018-03-14 10:30:42 +01:00
Frederik Hanghøj Iversen 7065455712 More readable goal for voevodsky's construction 2018-03-13 11:29:13 +01:00
Frederik Hanghøj Iversen fe453a6d3a Trying to prove cummulativity of homotopy levels 2018-03-12 16:00:27 +01:00
Frederik Hanghøj Iversen c52384b012 Change name of fromMonad 2018-03-12 14:43:43 +01:00
Frederik Hanghøj Iversen 5e092964c8 Change naming and fuse some modules 2018-03-12 14:38:52 +01:00
Frederik Hanghøj Iversen ccf753d438 Move monoidal and kleisli representation to own modules 2018-03-12 14:23:23 +01:00
Frederik Hanghøj Iversen aa645fb11e Move voevodsky's construction to own module 2018-03-12 14:04:10 +01:00