lean2/tests/lean/run/blast_cc5.lean

18 lines
587 B
Text
Raw Normal View History

set_option blast.strategy "cc"
example (a b c : Prop) : (a ↔ b) → ((a ∧ (c b)) ↔ (b ∧ (c a))) :=
by blast
/-
example (a b c : Prop) : (a ↔ b) → ((a ∧ (c (b ↔ a))) ↔ (b ∧ (c (a ↔ b)))) :=
by blast
example (a₁ a₂ b₁ b₂ : Prop) : (a₁ ↔ b₁) → (a₂ ↔ b₂) → (a₁ ∧ a₂ ∧ a₁ ∧ a₂ ↔ b₁ ∧ b₂ ∧ b₁ ∧ b₂) :=
by blast
definition lemma1 (a₁ a₂ b₁ b₂ : Prop) : (a₁ = b₁) → (a₂ ↔ b₂) → (a₁ ∧ a₂ ∧ a₁ ∧ a₂ ↔ b₁ ∧ b₂ ∧ b₁ ∧ b₂) :=
by blast
print lemma1
-/