mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-16 08:58:39 +00:00
13 lines
406 B
Agda
13 lines
406 B
Agda
{-# OPTIONS --safe --warning=error --without-K #-}
|
||
|
||
open import Functions
|
||
open import LogicalFormulae
|
||
open import Numbers.Naturals.Definition
|
||
open import Sets.Cardinality.Infinite.Definition
|
||
open import Sets.FinSet.Definition
|
||
|
||
module Sets.Cardinality.Infinite.Lemmas where
|
||
|
||
finsetNotInfinite : {n : ℕ} → InfiniteSet (FinSet n) → False
|
||
finsetNotInfinite {n} isInfinite = isInfinite n id idIsBijective
|