Skip to content

Commit

Permalink
qualify import
Browse files Browse the repository at this point in the history
  • Loading branch information
felixwellen committed Jan 25, 2024
1 parent b189e4a commit 1e9c959
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Cubical/Data/Nat/Triangular.agda
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ module Cubical.Data.Nat.Triangular where
open import Cubical.Foundations.Prelude
open import Cubical.Foundations.Function

open import Cubical.Data.FinData
open import Cubical.Data.FinData as Fin
open import Cubical.Data.Nat using (ℕ; suc; zero)

open import Cubical.Algebra.CommSemiring
Expand All @@ -22,7 +22,7 @@ first n i = toℕ i

firstDecompose : (n : ℕ) first (suc n) ∘ weakenFin ≡ first n
firstDecompose n i l =
elim
Fin.elim
(λ l first (suc _) (weakenFin l) ≡ first _ l)
refl
(λ _ weakenRespToℕ _)
Expand Down

0 comments on commit 1e9c959

Please sign in to comment.