2014-01-23 20:57:05 +00:00
|
|
|
|
rewrite_set simple
|
|
|
|
|
add_rewrite and_truer and_truel and_falser and_falsel or_falsel : simple
|
|
|
|
|
(*
|
|
|
|
|
add_congr_theorem("simple", "and_congr")
|
|
|
|
|
add_congr_theorem("simple", "or_congr")
|
|
|
|
|
*)
|
|
|
|
|
|
|
|
|
|
variables a b c : Nat
|
|
|
|
|
|
|
|
|
|
(*
|
|
|
|
|
local opts = options({"simplifier", "contextual"}, false)
|
|
|
|
|
local t = parse_lean([[a = 1 ∧ (¬ b = 0 ∨ c ≠ 0 ∨ b + c > a)]])
|
2014-01-27 23:02:05 +00:00
|
|
|
|
local s, pr = simplify(t, "simple", opts)
|
2014-01-23 20:57:05 +00:00
|
|
|
|
print(s)
|
|
|
|
|
print(pr)
|
|
|
|
|
print(get_environment():type_check(pr))
|
|
|
|
|
*)
|