lean2/tests/lean/run/blast_grind1.lean
Leonardo de Moura 17a2f1fe47 chore(tests/lean/run/blast_grind1): use 'core_grind'
Reason: we will change the semantics of 'grind'
2016-01-01 16:46:15 -08:00

32 lines
911 B
Text
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

set_option blast.strategy "core_grind"
example (a b c : nat) : a = b a = c → b = c → b = a :=
by blast
example (f : nat → nat) (a b c : nat) : f a = f b f a = f c → f b = f c → f b = f a :=
by blast
definition ex1 (a : nat) : a = 0 → (λ x, x + a) = (λ x, x + 0) :=
by blast
print ex1
attribute Exists.intro [intro!] -- core_grind only process [intro!] declarations
example (p q : nat → Prop) : (∃ x, p x ∧ q x) → (∃ x, q x) ∧ (∃ x, p x) :=
by blast
set_option blast.strategy "core_grind"
example (a b c : nat) : a = b a = c → b = c → b = a :=
by blast
example (f : nat → nat) (a b c : nat) : f a = f b f a = f c → f b = f c → f b = f a :=
by blast
example (a : nat) : a = 0 → (λ x, x + a) = (λ x, x + 0) :=
by blast
set_option trace.blast true
example (p q : nat → Prop) : (∃ x, p x ∧ q x) → (∃ x, q x) ∧ (∃ x, p x) :=
by blast