Revision 8a64c763e75234b20ddeb4c00839fa3eb92492cc authored by Bas Spitters on 27 October 2017, 16:07:50 UTC, committed by GitHub on 27 October 2017, 16:07:50 UTC
corn : switch to the external Bignums library
2 parent s 226b25a + 9e71c60
Raw File
Container.v
Require Import MathClasses.interfaces.canonical_names.

Class Container (Elem C: Type) := In: C → Elem → Prop.
Hint Unfold In.
Notation "x ∈ y" := (In y x) (at level 70).
Notation "x ∉ y" := (¬In y x) (at level 70).
Notation "(∈ y )" := (In y).
back to top