You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
{{ message }}
This repository has been archived by the owner on Oct 14, 2023. It is now read-only.
Reduced the issue to a self-contained, reproducible test case.
Description
@[simp]deffact (n : ℕ) : ℕ :=
nat.rec
1
(λ n' fact_n', (nat.succ n') * fact_n')
n
universe u
@[simp]defnat.rec_succ {P : ℕ → Type u} (o : P 0) (s : ∀ n, P n → P (nat.succ n)) (n : ℕ) : (nat.rec o s (nat.succ n) : P (nat.succ n)) = s n (nat.rec o s n) := rfl
example : fact 5 = 5 :=
begin
simp [fact,has_mul.mul,nat.mul],
rewrite [nat.rec_succ]
-- 15:3: failed-- state:-- ⊢ nat.rec 1 (λ (n' : ℕ), nat.mul (nat.succ n')) 5 = 5end
Expected behavior:rewrite succeeds
Actual behavior:rewrite fails
Reproduces how often: [What percentage of the time does it reproduce?] 100%
Versions
$ lean --version
Lean (version 3.4.2, commit cbd2b6686ddb, Release)
$ lsb_release -a
No LSB modules are available.
Distributor ID: Ubuntu
Description: Ubuntu 16.04.6 LTS
Release: 16.04
Codename: xenial
$ uname -a
Linux jgross-Leopard-WS 4.4.0-161-generic #189-Ubuntu SMP Tue Aug 27 08:10:16 UTC 2019 x86_64 x86_64 x86_64 GNU/Linux
The text was updated successfully, but these errors were encountered:
Prerequisites
or feature requests.
Description
Expected behavior:
rewrite
succeedsActual behavior:
rewrite
failsReproduces how often: [What percentage of the time does it reproduce?] 100%
Versions
The text was updated successfully, but these errors were encountered: