Free-group lemmas (#106)

This commit is contained in:
Patrick Stevens
2020-04-05 11:09:12 +01:00
committed by GitHub
parent 61b5f8acc5
commit 2f07a8e972
18 changed files with 327 additions and 188 deletions

View File

@@ -0,0 +1,16 @@
{-# OPTIONS --safe --warning=error --without-K #-}
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
open import Functions
open import Numbers.Naturals.Definition
open import Sets.FinSet.Definition
open import Setoids.Setoids
module Setoids.Cardinality.Finite.Definition where
record FiniteSetoid {a b : _} {A : Set a} (S : Setoid {a} {b} A) : Set (a b) where
field
size :
mapping : FinSet size A
bij : SetoidBijection (reflSetoid (FinSet size)) S mapping