This website requires JavaScript.
Explore
Help
Sign in
michael
/
lean2
Watch
1
Star
0
Fork
You've already forked lean2
0
Code
Issues
Pull requests
Projects
Releases
Packages
Wiki
Activity
Actions
37fdac4d65
lean2
/
tests
/
lean
/
run
/
blast_simp2.lean
5 lines
83 B
Text
Raw
Normal View
History
Unescape
Escape
feat(library/blast/simplifier/simplifier_actions): add simplify_hypothesis_action
2015-11-23 01:49:00 +00:00
definition tst1 (a b : Prop) : a ∧ b ∧ true → b ∧ a :=
test(tests/lean/run): use 'simp' when testing the simplifier
2015-12-06 22:35:14 +00:00
by simp
feat(library/blast/simplifier/simplifier_actions): add simplify_hypothesis_action
2015-11-23 01:49:00 +00:00
print tst1
Reference in a new issue
Copy permalink