Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

convert generates proof that is not accepted by the kernel #9805

Closed
gebner opened this issue Oct 19, 2021 · 3 comments
Closed

convert generates proof that is not accepted by the kernel #9805

gebner opened this issue Oct 19, 2021 · 3 comments
Labels
bug t-meta Tactics, attributes or user commands

Comments

@gebner
Copy link
Member

gebner commented Oct 19, 2021

import tactic

example : 1 = 0 :=
begin
  convert of_mul_one,
  apply_instance,
  -- goals accomplished!
end
@robertylewis robertylewis added bug t-meta Tactics, attributes or user commands labels Oct 19, 2021
@robertylewis
Copy link
Member

(To clarify for anyone who's reading this and worried, this is just a tactic bug. The proof is rejected by the type checker.)

@gebner gebner changed the title convert proves 1=0 convert generates proof that is not accepted by kernel Oct 27, 2021
@gebner gebner changed the title convert generates proof that is not accepted by kernel convert generates proof that is not accepted by the kernel Oct 27, 2021
@robertylewis
Copy link
Member

This goes up the food chain:

import algebra.group.type_tags 

lemma test2 : (0 : ℕ) = (0 : additive ℕ) := 
by tactic.reflexivity 

I don't have a mathlib-free MWE yet. Not sure what it is about additive that allows this.

@gebner
Copy link
Member Author

gebner commented Nov 1, 2021

Reported upstream as leanprover-community/lean#644

Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
bug t-meta Tactics, attributes or user commands
Projects
None yet
Development

No branches or pull requests

2 participants