Skip to content

Commit

Permalink
fixes
Browse files Browse the repository at this point in the history
  • Loading branch information
kbuzzard committed Oct 14, 2023
1 parent f625cb5 commit 3648e91
Show file tree
Hide file tree
Showing 2 changed files with 7 additions and 10 deletions.
5 changes: 0 additions & 5 deletions Game/Tactic/Induction.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,11 +3,6 @@ import Lean.Elab.Tactic.Induction
import Std.Tactic.OpenPrivate
import Std.Data.List.Basic
import Game.MyNat.Definition
import Lean
import Std.Tactic.OpenPrivate
import Std.Data.List.Basic
import Mathlib.Lean.Expr.Basic

import Mathlib.Lean.Expr.Basic


Expand Down
12 changes: 7 additions & 5 deletions Game/Tactic/cases_test.lean
Original file line number Diff line number Diff line change
@@ -1,18 +1,20 @@
import Game.Levels.LessOrEqual

namespace MyNat

example (P Q : Prop) (h : P ∨ Q) : False := by
cases h with hp hq
sorry -- hp : P
sorry -- hq : Q
· sorry -- hp : P
· sorry -- hq : Q

example (a b : ℕ) (h : a ≤ b) : False := by
cases h with c hc
-- hc: b = a + c
sorry

-- not working yet
example (a : ℕ) : a = a := by
cases a with d
-- get MyNat.zero because we used rec not rec' :-(
sorry

sorry
· sorry
· sorry

0 comments on commit 3648e91

Please sign in to comment.