HITs-Examples/FiniteSets/fsets/operations_cons_repr.v

19 lines
360 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.
Context {A : Type}.
Definition append (x y: FSetC A) : FSetC A.
hinduction x.
- apply y.
- apply Cns.
- apply dupl.
- apply comm.
Defined.
Definition singleton (a:A) : FSetC A := a;;.
End operations.