Skip to content

Commit 9021b2c

Browse files
committed
Test case for tests/lean/run/issue11449.lean
1 parent 9941e42 commit 9021b2c

File tree

2 files changed

+31
-2
lines changed

2 files changed

+31
-2
lines changed

tests/lean/run/issue11449.lean

Lines changed: 29 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,29 @@
1+
opaque double : Nat → Nat
2+
3+
inductive Parity : Nat -> Type
4+
| even (n) : Parity (double n)
5+
| odd (n) : Parity (Nat.succ (double n))
6+
7+
example
8+
(motive : (x : Nat) → Parity x → Sort u_1)
9+
(h_2 : (j : Nat) → motive (double j) (Parity.even j))
10+
(j n : Nat)
11+
(heq_1 : double n = double j)
12+
(heq_2 : Parity.even n ≍ Parity.even j):
13+
h_2 n ≍ h_2 j := by
14+
fail_if_success grind -- does not work yet
15+
sorry
16+
17+
-- manual proof using heterogenenous noConfusion
18+
19+
example
20+
(motive : (x : Nat) → Parity x → Sort u_1)
21+
(h_2 : (j : Nat) → motive (double j) (Parity.even j))
22+
(j n : Nat)
23+
(heq_1 : double n = double j)
24+
(heq_2 : Parity.even n ≍ Parity.even j):
25+
h_2 n ≍ h_2 j := by
26+
apply Parity.noConfusion heq_1 heq_2
27+
intro hnj
28+
subst hnj
29+
rfl

tests/lean/run/structuralMutual.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -512,13 +512,13 @@ Too many possible combinations of parameters of type Nattish (or please indicate
512512
Could not find a decreasing measure.
513513
The basic measures relate at each recursive call as follows:
514514
(<, ≤, =: relation proved, ? all proofs failed, _: no proof attempted)
515-
Call from ManyCombinations.f to ManyCombinations.g at 543:15-29:
515+
Call from ManyCombinations.f to ManyCombinations.g at 544:15-29:
516516
#1 #2 #3 #4
517517
#5 ? ? ? ?
518518
#6 ? ? = ?
519519
#7 ? ? ? =
520520
#8 ? = ? ?
521-
Call from ManyCombinations.g to ManyCombinations.f at 546:15-29:
521+
Call from ManyCombinations.g to ManyCombinations.f at 547:15-29:
522522
#5 #6 #7 #8
523523
#1 _ _ _ _
524524
#2 _ _ _ ?

0 commit comments

Comments
 (0)