1
0
mirror of https://github.com/nmvdw/HITs-Examples synced 2025-12-24 18:23:51 +01:00
Files
HITs-Examples/FiniteSets/fsets/operations_cons_repr.v
2017-08-08 17:00:30 +02:00

18 lines
421 B
Coq

(* Operations on [FSetC A] *)
Require Import HoTT HitTactics.
Require Import representations.cons_repr.
Section operations.
Global Instance fsetc_union : forall A, hasUnion (FSetC A).
Proof.
intros A x y.
hinduction x.
- apply y.
- apply Cns.
- apply dupl.
- apply comm.
Defined.
Global Instance fsetc_singleton : forall A, hasSingleton (FSetC A) A := fun A a => a;;.
End operations.