Skip to content

Commit

Permalink
split cumulative hierarchy
Browse files Browse the repository at this point in the history
  • Loading branch information
WorldSEnder committed Oct 2, 2020
1 parent 8097c1a commit 37c526c
Show file tree
Hide file tree
Showing 4 changed files with 504 additions and 441 deletions.
6 changes: 6 additions & 0 deletions Cubical/HITs/CumulativeHierarchy.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,6 @@
{-# OPTIONS --cubical --no-import-sorts --safe #-}
module Cubical.HITs.CumulativeHierarchy where

open import Cubical.HITs.CumulativeHierarchy.Base public
open import Cubical.HITs.CumulativeHierarchy.Properties public
open import Cubical.HITs.CumulativeHierarchy.Constructions public
Loading

0 comments on commit 37c526c

Please sign in to comment.