summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/1901.v
blob: 598db36601f66d5e5ba00bd23127777ed213dc30 (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.