blob: 7d86adbfb28f09139ba0dcda6dbc68cbd4d22106 (
plain)
1
2
3
4
5
6
7
8
9
10
11
|
Require Import Relations.
Record Poset{A:Type}(Le : relation A) : Type :=
Build_Poset
{
Le_refl : forall x : A, Le x x;
Le_trans : forall x y z : A, Le x y -> Le y z -> Le x z;
Le_antisym : forall x y : A, Le x y -> Le y x -> x = y }.
Definition nat_Poset : Poset Peano.le.
Admitted.
|