Skip to content

Commit

Permalink
fixed some imports
Browse files Browse the repository at this point in the history
  • Loading branch information
Saizan committed Dec 29, 2017
1 parent 62a3287 commit cc4bcc4
Show file tree
Hide file tree
Showing 7 changed files with 31 additions and 19 deletions.
27 changes: 15 additions & 12 deletions examples/Cubical/Examples/Category.agda
Original file line number Diff line number Diff line change
@@ -1,7 +1,8 @@
{-# OPTIONS --cubical #-}
module Cubical.Examples.Category where

open import PathPrelude
open import Cubical.FromStdLib
open import Cubical.PathPrelude

-- Functor
record Func {ℓ} : Set (ℓ-suc ℓ) where
Expand Down Expand Up @@ -56,19 +57,21 @@ G ∘ᶠ F = record
module G = Func G

idᶠLeft : {ℓ}{F : Func {ℓ}} idᶠ ∘ᶠ F ≡ F
idᶠLeft {ℓ} {F} = Func≡.path r where
idᶠLeft {ℓ} {F} =
directpath where
-- Func≡.path r where
module L = Func (idᶠ ∘ᶠ F)
module R = Func F
map≡ : L.map ≡ R.map
map≡ = funExt (λ _ refl)
r = record { F = idᶠ ∘ᶠ F
; G = F
; map≡ = λ A refl
; fmap≡ = λ f funExt λ _ refl
; presId≡ = λ A {!!}
; presComp≡ = λ f g {!!}
}
open import Comp
-- map≡ : L.map ≡ R.map
-- map≡ = funExt (λ _ → refl)
-- r = record { F = idᶠ ∘ᶠ F
-- ; G = F
-- ; map≡ = λ A → refl
-- ; fmap≡ = λ f → funExt λ _ → refl
-- ; presId≡ = λ A → {!!}
-- ; presComp≡ = λ f g → {!!}
-- }
open import Cubical.Comp as Comp

trans-id : {ℓ}{A : Set ℓ} {x y : A} (p : x ≡ y) trans p (\ i y) ≡ p
trans-id {A = A} {x} {y} p i j = Comp.fill (λ _ A) _
Expand Down
1 change: 1 addition & 0 deletions examples/Cubical/Examples/Cube.agda
Original file line number Diff line number Diff line change
Expand Up @@ -3,6 +3,7 @@ module Cubical.Examples.Cube where

open import Cubical.PathPrelude
open import Cubical.Id
open import Cubical.FromStdLib

test-sym : {ℓ} {A : Set ℓ} {x y : A} (p : x ≡ y) sym (sym p) ≡ p
test-sym p = refl
Expand Down
6 changes: 6 additions & 0 deletions examples/Cubical/Examples/Everything.agda
Original file line number Diff line number Diff line change
Expand Up @@ -14,6 +14,12 @@ open import Cubical.Examples.Cube
open import Cubical.Examples.OTTU

open import Cubical.Examples.BinNat
open import Cubical.Examples.Int
open import Cubical.Examples.SizedStream

open import Cubical.Examples.Category
open import Cubical.Examples.FunctorCWF


-- Demo
open import Cubical.Examples.AIM_Demo.DemoPath
Expand Down
5 changes: 3 additions & 2 deletions examples/Cubical/Examples/FunctorCWF.agda
Original file line number Diff line number Diff line change
@@ -1,7 +1,8 @@
{-# OPTIONS --cubical #-}
module FunctorCWF where
module Cubical.Examples.FunctorCWF where

open import PathPrelude hiding (_∘_)
open import Cubical.PathPrelude
open import Cubical.FromStdLib hiding (_∘_)

Σ= : {a b} {A : Set a} {B : A Set b} {x y : Σ A B} (eq : x .fst ≡ y .fst)
PathP (\ i B (eq i)) (x .snd) (y .snd) x ≡ y
Expand Down
1 change: 1 addition & 0 deletions examples/Cubical/Examples/OTTU.agda
Original file line number Diff line number Diff line change
Expand Up @@ -2,6 +2,7 @@
module Cubical.Examples.OTTU where

open import Cubical.PathPrelude
open import Cubical.FromStdLib

open import Cubical.Examples.Cube

Expand Down
8 changes: 4 additions & 4 deletions examples/Cubical/Examples/SizedStream.agda
Original file line number Diff line number Diff line change
@@ -1,9 +1,9 @@
{-# OPTIONS --cubical #-}
module SizedStream where
module Cubical.Examples.SizedStream where

open import Data.Product using (_×_)
open import PathPrelude
open import Size
open import Cubical.PathPrelude
open import Cubical.FromStdLib using (_×_)
open import Agda.Builtin.Size

record Stream (A : Set) (i : Size) : Set where
coinductive
Expand Down
2 changes: 1 addition & 1 deletion examples/Cubical/Examples/Stream.agda
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@

module Cubical.Examples.Stream where

open import Cubical.FromStdLib using (_×_)
open import Cubical.FromStdLib using (_×_; ℕ; zero; suc)
open import Cubical.PathPrelude


Expand Down

0 comments on commit cc4bcc4

Please sign in to comment.