HITs-Examples/FiniteSets/fsets/operations_cons_repr.v

18 lines
421 B
Coq
Raw Normal View History

2017-08-02 11:40:03 +02:00
(* Operations on [FSetC A] *)
Require Import HoTT HitTactics.
Require Import representations.cons_repr.
Section operations.
2017-08-08 17:00:30 +02:00
Global Instance fsetc_union : forall A, hasUnion (FSetC A).
2017-08-08 15:29:50 +02:00
Proof.
intros A x y.
2017-08-02 11:40:03 +02:00
hinduction x.
- apply y.
- apply Cns.
- apply dupl.
- apply comm.
Defined.
2017-08-08 17:00:30 +02:00
Global Instance fsetc_singleton : forall A, hasSingleton (FSetC A) A := fun A a => a;;.
2017-08-02 11:40:03 +02:00
End operations.