Skip to content

Commit

Permalink
make simp_add available in the entire game #54
Browse files Browse the repository at this point in the history
  • Loading branch information
joneugster committed Mar 18, 2024
1 parent 61ce832 commit c35d29d
Show file tree
Hide file tree
Showing 5 changed files with 40 additions and 395 deletions.
1 change: 1 addition & 0 deletions Game/Levels/Algorithm/L04add_algo3.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
import Game.Levels.Algorithm.L03add_algo2
import ImportGraph

World "Algorithm"
Level 4
Expand Down
5 changes: 1 addition & 4 deletions Game/Metadata.lean
Original file line number Diff line number Diff line change
Expand Up @@ -14,10 +14,7 @@ import Game.Tactic.Rw
import Game.Tactic.Use
import Game.Tactic.Ne
import Game.Tactic.Xyzzy
import Game.Tactic.SimpAdd
-- import Std.Tactic.RCases
-- import Game.Tactic.Have
-- import Game.Tactic.LeftRight

-- TODO: Why does this not work here??
-- We do not want `simp` to be able to do anything unless we unlock it manually.
attribute [-simp] MyNat.succ.injEq
342 changes: 0 additions & 342 deletions Game/Tactic/LeanExprBasic.lean

This file was deleted.

Loading

0 comments on commit c35d29d

Please sign in to comment.