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