hbhb bbk
$$ ref\ U\ R:=\forall x:U,R \ x\ x $$
$$ total\ U\ R:=\forall x\ y,R\ x\ y\lor R\ y \ x\ $$
$$ \forall U(R:U\rightarrow U\rightarrow Prop),total\ R\rightarrow ref \ R $$
Require Import Utf8.
Set Implicit Arguments.
Definition imp(a b:Prop):=a → b.
Definition ref U R:=∀x:U,R x x.
Definition total U R:=∀x y:U,R x y∨R y x.
Goal ∀U(R:U → U → Prop),total R → ref R.
Abort.