test(tests/lean/run): use 'simp' when testing the simplifier
This commit is contained in:
parent
67e291ac84
commit
5626431c7f
3 changed files with 8 additions and 18 deletions
|
@ -1,17 +1,17 @@
|
|||
example (a b c : Prop) : a ∧ b ∧ c ↔ c ∧ b ∧ a :=
|
||||
by blast
|
||||
by simp
|
||||
|
||||
example (a b c : Prop) : a ∧ false ∧ c ↔ false :=
|
||||
by blast
|
||||
by simp
|
||||
|
||||
example (a b c : Prop) : a ∨ false ∨ b ↔ b ∨ a :=
|
||||
by blast
|
||||
by simp
|
||||
|
||||
example (a b c : Prop) : ¬ true ∨ false ∨ b ↔ b :=
|
||||
by blast
|
||||
by simp
|
||||
|
||||
example (a b c : Prop) : if true then a else b ↔ if false then b else a :=
|
||||
by blast
|
||||
by simp
|
||||
|
||||
example (a b : Prop) : a ∧ not a ↔ false :=
|
||||
by blast
|
||||
by simp
|
||||
|
|
|
@ -1,6 +1,4 @@
|
|||
set_option blast.recursor false
|
||||
|
||||
definition tst1 (a b : Prop) : a ∧ b ∧ true → b ∧ a :=
|
||||
by blast
|
||||
by simp
|
||||
|
||||
print tst1
|
||||
|
|
|
@ -1,11 +1,3 @@
|
|||
set_option blast.simp false
|
||||
|
||||
example (A : Type₁) (a₁ a₂ : A) : a₁ = a₂ →
|
||||
(λ (B : Type₁) (f : A → B), f a₁) = (λ (B : Type₁) (f : A → B), f a₂) :=
|
||||
by blast
|
||||
|
||||
set_option blast.simp true
|
||||
|
||||
example (A : Type₁) (a₁ a₂ : A) : a₁ = a₂ →
|
||||
(λ (B : Type₁) (f : A → B), f a₁) = (λ (B : Type₁) (f : A → B), f a₂) :=
|
||||
by blast
|
||||
by simp
|
||||
|
|
Loading…
Reference in a new issue