Library mathcomp.boot.ssrbool

From mathcomp Require Import ssreflect ssrfun.
From Corelib Require Export ssrbool.
Set Implicit Arguments.

not yet backported

Lemma homo_mono1 [aT rT : Type] [f : aT rT] [g : rT aT]
    [aP : pred aT] [rP : pred rT] :
  cancel g f
  {homo f : x / aP x >-> rP x}
  {homo g : x / rP x >-> aP x} {mono g : x / rP x >-> aP x}.

Lemma if_and b1 b2 T (x y : T) :
  (if b1 && b2 then x else y) = (if b1 then if b2 then x else y else y).

Lemma if_or b1 b2 T (x y : T) :
  (if b1 || b2 then x else y) = (if b1 then x else if b2 then x else y).

Lemma if_implyb b1 b2 T (x y : T) :
  (if b1 ==> b2 then x else y) = (if b1 then if b2 then x else y else x).

Lemma if_implybC b1 b2 T (x y : T) :
  (if b1 ==> b2 then x else y) = (if b2 then x else if b1 then y else x).

Lemma if_add b1 b2 T (x y : T) :
  (if b1 (+) b2 then x else y) = (if b1 then if b2 then y else x else if b2 then x else y).

Lemma relpre_trans {T' T : Type} {leT : rel T} {f : T' T} :
  transitive leT transitive (relpre f leT).