Skip to content

Commit dda69b3

Browse files
committed
Disable in some tests
1 parent 92a89ce commit dda69b3

File tree

7 files changed

+24
-7
lines changed

7 files changed

+24
-7
lines changed

src/Lean/Meta/Match/Match.lean

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -330,8 +330,10 @@ private abbrev isCtorIdxIneq? (e : Expr) : Option FVarId := do
330330

331331
private partial def contradiction (mvarId : MVarId) : MetaM Bool := do
332332
mvarId.withContext do
333-
trace[Meta.Match.match] "match contradiction:\n{mvarId}"
333+
withTraceNode `Meta.Match.match (msg := (return m!"{exceptBoolEmoji ·} Match.contradiction")) do
334+
trace[Meta.Match.match] m!"Match.contradiction:\n{mvarId}"
334335
if (← mvarId.contradictionCore {}) then
336+
trace[Meta.Match.match] "Contradiction found!"
335337
return true
336338
else
337339
-- Try harder by splitting `ctorIdx x ≠ 23` assumptions
@@ -587,7 +589,7 @@ private def processConstructor (p : Problem) : MetaM (Array Problem) := do
587589
else
588590
-- A catch-all case
589591
let subst := subgoal.subst
590-
trace[Meta.Match.match] "constructor catch-all case. subst: {subst.map.toList.map fun p => (mkFVar p.1, p.2)}"
592+
trace[Meta.Match.match] "constructor catch-all case"
591593
let examples := p.examples.map <| Example.applyFVarSubst subst
592594
let newVars := p.vars.map fun x => x.applyFVarSubst subst
593595
let newAlts := p.alts.filter fun alt => match alt.patterns with
Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,2 +1,2 @@
11
matchErrorMsg.lean:2:1-2:6: error: Missing cases:
2-
(Prod.mk Nat.zero (Nat.succ _))
2+
(Prod.mk Nat.zero _)

tests/lean/matchUnknownFVarBug.lean.expected.out

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,8 +1,8 @@
11
matchUnknownFVarBug.lean:2:2-2:7: error: Missing cases:
2-
(some (Nat.succ _)), (some _)
3-
(some (Nat.succ _)), none
42
none, (some _)
53
none, none
4+
(some _), (some _)
5+
(some _), none
66
matchUnknownFVarBug.lean:3:18-3:19: error: unsolved goals
77
n? x✝ : Option Nat
88
h : n? = some 0
Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
patvar.lean:3:0-3:22: error: Missing cases:
2-
(List.cons _ _)
2+
_
33
patvar.lean:10:0-10:16: error: Missing cases:
4-
(List.cons _ _)
4+
_
55
patvar.lean:14:2-14:9: error: Invalid pattern variable: Variable name must be atomic, but `foo.bar` has multiple components
66
patvar.lean:17:2-17:9: error: Invalid pattern variable: Variable name must be atomic, but `foo.bar` has multiple components

tests/lean/run/bv_decide_enum_universe.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -65,6 +65,7 @@ def test4 (x : PBool.{1}) : Bool :=
6565
| .false => false
6666
| .true => false
6767

68+
set_option match.use_sparse_cases false -- TODO
6869
def test5 (x : PBool) : Bool :=
6970
match x with
7071
| .true => false

tests/lean/run/bv_decide_enums_two.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,7 @@ inductive State : Type
44
| A : State
55
| B : State
66

7+
set_option match.use_sparse_cases false
78

89
def myFunc (s : State) : Bool :=
910
match s with

tests/lean/run/match_int_lit_issue.lean

Lines changed: 13 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,16 @@
1+
set_option match.use_sparse_cases false -- TODO
2+
-- set_option trace.Meta.Match.match true
3+
4+
/-
5+
This breaks because of less case splitting, and moving the case splitting to
6+
the contradiction phase is not enough, as `contradiction` does not look more than
7+
one constructor deep:
8+
```
9+
example (n : Nat) (h : n.succ = 0) : False := by contradiction
10+
example (n : Nat) (h : Int.ofNat n.succ = 0) : False := by contradiction
11+
```
12+
-/
13+
114
theorem Int.eq_zero_of_sign_eq_zero' : ∀ {a : Int}, sign a = 0 → a = 0
215
| 0, _ => rfl
316

0 commit comments

Comments
 (0)