File tree Expand file tree Collapse file tree 1 file changed +2
-2
lines changed
Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -41,7 +41,7 @@ public theorem trichotomous_of_rel_or_eq_or_rel_swap {r : α → α → Prop}
4141 (h : ∀ {a b}, r a b ∨ a = b ∨ r b a) : Trichotomous r where
4242 trichotomous _ _ hab hba := (h.resolve_left hab).resolve_right hba
4343
44- public theorem Antisymm.trichotomous_of_antisymm_not {r : α → α → Prop } [i : Antisymm (¬ r · ·)] :
44+ public instance Antisymm.trichotomous_of_antisymm_not {r : α → α → Prop } [i : Antisymm (¬ r · ·)] :
4545 Trichotomous r where trichotomous := i.antisymm
4646
4747public theorem Trichotomous.antisymm_not {r : α → α → Prop } [i : Trichotomous r] :
@@ -62,7 +62,7 @@ public theorem total_of_refl_of_trichotomous (r : α → α → Prop) [Refl r] [
6262public theorem asymm_of_irrefl_of_antisymm (r : α → α → Prop ) [Irrefl r] [Antisymm r] :
6363 Asymm r where asymm a b h h' := Irrefl.irrefl _ (Antisymm.antisymm a b h h' ▸ h)
6464
65- public theorem Total.asymm_of_total_not {r : α → α → Prop } [i : Total (¬ r · ·)] : Asymm r where
65+ public instance Total.asymm_of_total_not {r : α → α → Prop } [i : Total (¬ r · ·)] : Asymm r where
6666 asymm a b h := (i.total a b).resolve_left (· h)
6767
6868public theorem Asymm.total_not {r : α → α → Prop } [i : Asymm r] : Total (¬ r · ·) where
You can’t perform that action at this time.
0 commit comments