Documentation

Logic.Modal.Standard.Kripke.Grz

def irreflexivize {α : Sort u_1} (R : ααProp) (x : α) (y : α) :
Equations
Instances For
    @[reducible, inline]
    abbrev WeaklyConverseWellFounded {α : Type u_1} (R : ααProp) :
    Equations
    Instances For
      theorem dependent_choice {α : Type u_1} {R : ααProp} (h : ∃ (s : Set α), s.Nonempty as, bs, R a b) :
      ∃ (f : α), ∀ (x : ), R (f x) (f (x + 1))
      theorem antisymm_of_WCWF :
      ∀ {α : Type u_1} {R : ααProp}, WeaklyConverseWellFounded RAntisymmetric R
      theorem Finite.exists_ne_map_eq_of_infinite_lt {α : Type u_1} {β : Sort u_2} [LinearOrder α] [Infinite α] [Finite β] (f : αβ) :
      ∃ (x : α) (y : α), x < y f x = f y
      theorem WCWF_of_antisymm_trans {α : Type u_1} {R : ααProp} (hFin : Finite α) (R_trans : Transitive R) :