2015-12-06 22:33:21 +00:00
|
|
|
set_option blast.strategy "cc"
|
2015-11-21 22:43:51 +00:00
|
|
|
|
|
|
|
example (a b c d : Prop)
|
|
|
|
[d₁ : decidable a] [d₂ : decidable b] [d₃ : decidable c] [d₄ : decidable d]
|
|
|
|
: (a ↔ b) → (c ↔ d) → ((if (a ∧ c) then true else false) ↔ (if (b ∧ d) then true else false)) :=
|
|
|
|
by blast
|
|
|
|
|
|
|
|
example (a b c d : Prop) (x y z : nat)
|
|
|
|
[d₁ : decidable a] [d₂ : decidable b] [d₃ : decidable c] [d₄ : decidable d]
|
|
|
|
: (a ↔ b) → (c ↔ d) → x = y → ((if (a ∧ c ∧ a) then x else y) = (if (b ∧ d ∧ b) then y else x)) :=
|
|
|
|
by blast
|