Skip to content

Commit

Permalink
clean up
Browse files Browse the repository at this point in the history
  • Loading branch information
mzhang28 committed Dec 6, 2024
1 parent 07c87ff commit 6363fa4
Showing 1 changed file with 0 additions and 3 deletions.
3 changes: 0 additions & 3 deletions Cubical/Algebra/Group/Exact.agda
Original file line number Diff line number Diff line change
Expand Up @@ -30,9 +30,6 @@ private
variable
ℓ ℓ' : Level

SuccStr : Type (ℓ-suc ℓ)
SuccStr {ℓ = ℓ} = TypeWithStr ℓ λ A (A A)

-- Exactness except the intersecting Group is only propositionally equal
isWeakExactAt : {A B B' C : Group ℓ} (f : GroupHom A B) (g : GroupHom B' C) (p : B ≡ B') Type ℓ
isWeakExactAt {ℓ = ℓ} {B = B} {B' = B'} f g p = (b : ⟨ B ⟩) (isInKer g (tr b) isInIm f b) × (isInIm f b isInKer g (tr b)) where
Expand Down

0 comments on commit 6363fa4

Please sign in to comment.