2014-09-09 15:04:44 -07:00
|
|
|
|
import logic
|
|
|
|
|
open decidable
|
|
|
|
|
|
2015-02-24 14:09:20 -08:00
|
|
|
|
definition decidable_bin_rel [reducible] {A : Type} (R : A → A → Prop) := Πx y, decidable (R x y)
|
2014-09-09 15:04:44 -07:00
|
|
|
|
|
|
|
|
|
section
|
2014-10-09 07:13:06 -07:00
|
|
|
|
variable {A : Type}
|
|
|
|
|
variable (R : A → A → Prop)
|
2014-09-09 15:04:44 -07:00
|
|
|
|
|
|
|
|
|
theorem tst1 (H : Πx y, decidable (R x y)) (a b c : A) : decidable (R a b ∧ R b a)
|
|
|
|
|
|
2014-09-09 16:07:07 -07:00
|
|
|
|
theorem tst2 (H : decidable_bin_rel R) (a b c : A) : decidable (R a b ∧ R b a ∨ R b b) :=
|
|
|
|
|
_
|
2014-09-09 15:04:44 -07:00
|
|
|
|
end
|