mirror of
https://github.com/nmvdw/HITs-Examples
synced 2025-12-15 22:53:51 +01:00
Uses merely decidable equality, added length.
This commit is contained in:
@@ -2,6 +2,10 @@
|
||||
Require Import HoTT HitTactics.
|
||||
Require Import kuratowski.kuratowski_sets.
|
||||
|
||||
(** We prove extensionality via a chain of equivalences.
|
||||
We end with proving that equality can be defined with the subset relation.
|
||||
From that we can conclude that [FSet A] has decidable equality if [A] has.
|
||||
*)
|
||||
Section ext.
|
||||
Context {A : Type}.
|
||||
Context `{Univalence}.
|
||||
|
||||
Reference in New Issue
Block a user