Zulip Chat Archive
Stream: general
Topic: Default proofs
Yaël Dillies (Sep 13 2021 at 21:14):
So I know how I can provide default arguments to fields of a class, but how can I provide default proofs about them? I know that for nsmul we use a tactic, which makes me fear I can't write a default as I would have wanted to.
Here's what I'm working on (wink wink Anne):
import data.finset.basic
class locally_finite_order (α : Type*) [preorder α] [decidable_rel ((≤) : α → α → Prop)] :=
(finset_Icc : α → α → finset α)
(finset_Ico : α → α → finset α := λ a b, (finset_Icc a b).filter (λ x, ¬b ≤ x))
(finset_Ioc : α → α → finset α := λ a b, (finset_Icc a b).filter (λ x, ¬a ≤ x))
(finset_Ioo : α → α → finset α := λ a b, (finset_Icc a b).filter (λ x, ¬a ≤ x ∧ ¬b ≤ x))
(finset_mem_Icc : ∀ a b x : α, x ∈ finset_Icc a b ↔ a ≤ x ∧ x ≤ b)
(finset_mem_Ico : ∀ a b x : α, x ∈ finset_Ico a b ↔ a ≤ x ∧ x ≤ b :=  λ a b x, begin
  -- I would like to replace `finset_Ico` by `(finset_Icc a b).filter (λ x, ¬a ≤ x)`
end)
(finset_mem_Ioc : ∀ a b x : α, x ∈ finset_Ioc a b ↔ a ≤ x ∧ x ≤ b)
(finset_mem_Ioo : ∀ a b x : α, x ∈ finset_Ioo a b ↔ a ≤ x ∧ x ≤ b)
Yury G. Kudryashov (Sep 13 2021 at 21:20):
Indeed, you can only use := default_val syntax if default_val works always, not only for default arguments.
Yury G. Kudryashov (Sep 13 2021 at 21:21):
You can create a bunch of lemmas, write a tactic meta def mytac := [apply_rules [my_lemmas]], then use . mytac`.
Yaël Dillies (Sep 13 2021 at 21:24):
Should be pretty easy here!
Yaël Dillies (Sep 13 2021 at 21:24):
But that's disappointing Lean doesn't allow that. Is there any technical limitation?
Mario Carneiro (Sep 13 2021 at 21:30):
Yes, the field has to be type correct
Mario Carneiro (Sep 13 2021 at 21:31):
I suppose you could call that a technical limitation
Yaël Dillies (Sep 13 2021 at 21:31):
Hmm... :thinking:
Mario Carneiro (Sep 13 2021 at 21:32):
The standard workaround for this is to use tactics instead, like Yury says. For example see the lt fields in docs#preorder
Yaël Dillies (Sep 13 2021 at 21:32):
The technical limitation rather sounds like you can't "undefault" a field that depends on another default field that's been provided by the user.
Mario Carneiro (Sep 13 2021 at 21:32):
order_laws_tac is just intros; refl
Mario Carneiro (Sep 13 2021 at 21:33):
Exactly; you would be in trouble if you have def foo (a := 1) (b : a = 1 := rfl) and then decided to use foo 2 _
Mario Carneiro (Sep 13 2021 at 21:34):
or more to the point, @foo 2
Mario Carneiro (Sep 13 2021 at 21:34):
which has the type \forall  (b : 2 = 1 := rfl), ... which doesn't typecheck
Yaël Dillies (Sep 13 2021 at 21:34):
I guess I don't know how default arguments work.
Mario Carneiro (Sep 13 2021 at 21:35):
A default argument (a : nat := 1) is just sugar for (a : opt_param nat 1)
Yaël Dillies (Sep 13 2021 at 21:35):
I guess I don't know how out_param works :rofl:
Mario Carneiro (Sep 13 2021 at 21:35):
and the type signature of docs#opt_param makes it clear that you can't put a default value that doesn't match the type
Mario Carneiro (Sep 13 2021 at 21:36):
that is, opt_param (2 = 1) rfl doesn't typecheck because rfl : 2 = 1 fails
Mario Carneiro (Sep 13 2021 at 21:36):
this is before we've even used the definition, mind
Yaël Dillies (Sep 13 2021 at 21:37):
Urf, yeah
Mario Carneiro (Sep 13 2021 at 21:38):
using tactics ("auto_param") works around this because we don't try to elaborate it until the definition is used
Kevin Buzzard (Sep 13 2021 at 21:39):
Yaël Dillies said:
I guess I don't know how
out_paramworks :rofl:
@[reducible] def out_param (α : Sort u) : Sort u := α
What could be simpler? It's just id!
Mario Carneiro (Sep 13 2021 at 21:39):
unfortunately you can't actually specify a tactic block in lean 3 (lean 4 lets you do this) because tactic is meta so terms of that type can't appear in definitions, so instead you have to specify the name of a tactic like order_laws_tac
Mario Carneiro (Sep 13 2021 at 21:40):
which is the reason for all the indirection
Mario Carneiro (Sep 13 2021 at 21:40):
actually that's out_param, not opt_param
Mario Carneiro (Sep 13 2021 at 21:40):
opt_param is only slightly more complicated:
@[reducible] def opt_param (α : Sort u) (default : α) : Sort u := α
Kevin Buzzard (Sep 13 2021 at 21:42):
In maths we call that
Kevin Buzzard (Sep 13 2021 at 21:43):
It was when you were working on modules a few years ago that it all dawned on me that stuff like id can be harder than it looks.
Eric Wieser (Sep 13 2021 at 23:57):
When does the elaborator populate an opt_param with its default vs leaving it as a binder?
Mario Carneiro (Sep 14 2021 at 00:08):
If it is a regular application f a b and the third argument is c := ... then it will insert the default value
Mario Carneiro (Sep 14 2021 at 00:09):
basically, if there are any pis left over in a regular application and they are auto/opt params then it will insert them
Mario Carneiro (Sep 14 2021 at 00:11):
Unlike implicits and typeclass args, they don't work if used out of order:
def foo (a := 1) (b : ℕ) := 1
#check foo _ 3 -- foo ?M_1 3 : ℕ
Mario Carneiro (Sep 14 2021 at 00:11):
If you use @foo or @@foo then it will disable all argument insertion
Yaël Dillies (Sep 14 2021 at 08:28):
Mario Carneiro said:
using tactics ("auto_param") works around this because we don't try to elaborate it until the definition is used
Why can't this be the default behavior?
Yaël Dillies (Sep 14 2021 at 08:40):
Also, I tried the customized tactic trick, but I'm stuck because I can't reproduce the state that the tactic must solve. With the same example as above, if I do not provide finset_Ico, I get in finset_mem_Ico the goal I expect except for the fact that finset_Icc has been replaced by its definition (which stops me from using finset_mem_Icc). But when I do not provide finset_mem_Ico either, my tactic sees a goal where finset_Ico nor  finset_Icc have been replaced by their definitions, but unfold locally_finite_order.finset_Ico or rw locally_finite_order.finset_Icowon't do anything.
Yaël Dillies (Sep 14 2021 at 08:42):
/me is writing a MWE
Yaël Dillies (Sep 14 2021 at 10:00):
I don't understand what's happening in either case.
import data.set.finite
section tactic
open tactic
meta def finset_Ico_laws_tac : tactic unit :=
whnf_target >> intros >> to_expr``(begin
  unfold locally_finite_order.finset_Ico,
  rw [finset.mem_filter, finset_mem_Icc, and_assoc, lt_iff_le_not_le]
end) >>= exact
end tactic
open finset
class locally_finite_order (α : Type*) [preorder α] [decidable_rel ((≤) : α → α → Prop)] :=
(finset_Icc : α → α → finset α)
(finset_Ico : α → α → finset α := λ a b, (finset_Icc a b).filter (λ x, ¬b ≤ x))
(finset_mem_Icc : ∀ a b x : α, x ∈ finset_Icc a b ↔ a ≤ x ∧ x ≤ b)
(finset_mem_Ico : ∀ a b x : α, x ∈ finset_Ico a b ↔ a ≤ x ∧ x < b . finset_Ico_laws_tac)
variables {α : Type*} [preorder α] [decidable_rel ((≤) : α → α → Prop)]
noncomputable def locally_finite_order_of_finite_Icc'
  (h : ∀ a b : α, (set.Icc a b).finite) :
  locally_finite_order α :=
{ finset_Icc := λ a b, (h a b).to_finset,
  finset_mem_Icc := λ a b x, by rw [set.finite.mem_to_finset, set.mem_Icc] }
/-simplify tactic failed to simplify
state:
α : Type u_1,
_inst_1 : preorder α,
_inst_2 : decidable_rel has_le.le,
h : ∀ (a b : α), (set.Icc a b).finite,
a b x : α
⊢ ?m_1
state:
α : Type u_1,
_inst_1 : preorder α,
_inst_2 : decidable_rel has_le.le,
h : ∀ (a b : α), (set.Icc a b).finite,
a b x : α
⊢ x ∈ filter (λ (x : α), ¬preorder.le b x) _.to_finset ↔ a ≤ x ∧ x < b-/
noncomputable def locally_finite_order_of_finite_Icc
  (h : ∀ a b : α, (set.Icc a b).finite) :
  locally_finite_order α :=
{ finset_Icc := λ a b, (h a b).to_finset,
  finset_mem_Icc := λ a b x, by rw [set.finite.mem_to_finset, set.mem_Icc],
  finset_mem_Ico := λ a b x, begin
    rw [finset.mem_filter, finset_mem_Icc, and_assoc, lt_iff_le_not_le], -- finset_mem_Icc
  end }
Yaël Dillies (Sep 14 2021 at 17:21):
Bump! Has anybody ideas?
Yaël Dillies (Sep 14 2021 at 17:24):
I switched to change and it seems more reliable, but I'm still blindcoding
Mario Carneiro (Sep 14 2021 at 19:14):
Why don't you just write a lemma instead of reproving the lemma every time someone uses your theorem?
Mario Carneiro (Sep 14 2021 at 19:31):
Hm, this has the unfortunate requirement that it needs finset_mem_Icc to be a hypothesis in scope, so you have to write the thing a little weirdly if you want to avoid repeating yourself:
import data.set.finite
theorem locally_finite_order.mem_Ico_of_mem_Icc
  {α : Type*} [preorder α] [decidable_rel ((≤) : α → α → Prop)]
  {finset_Icc : α → α → finset α}
  (finset_mem_Icc : ∀ a b x : α, x ∈ finset_Icc a b ↔ a ≤ x ∧ x ≤ b)
  (a b x : α) : x ∈ (finset_Icc a b).filter (λ x, ¬b ≤ x) ↔ a ≤ x ∧ x < b :=
by rw [finset.mem_filter, finset_mem_Icc, and_assoc, lt_iff_le_not_le]
meta def finset_Ico_laws_tac : tactic unit :=
`[exact locally_finite_order.mem_Ico_of_mem_Icc finset_mem_Icc]
class locally_finite_order (α : Type*) [preorder α] [decidable_rel ((≤) : α → α → Prop)] :=
(finset_Icc : α → α → finset α)
(finset_Ico : α → α → finset α := λ a b, (finset_Icc a b).filter (λ x, ¬b ≤ x))
(finset_mem_Icc : ∀ a b x : α, x ∈ finset_Icc a b ↔ a ≤ x ∧ x ≤ b)
(finset_mem_Ico : ∀ a b x : α, x ∈ finset_Ico a b ↔ a ≤ x ∧ x < b . finset_Ico_laws_tac)
variables {α : Type*} [preorder α] [decidable_rel ((≤) : α → α → Prop)]
noncomputable def locally_finite_order_of_finite_Icc'
  (h : ∀ a b : α, (set.Icc a b).finite) :
  locally_finite_order α :=
begin
  suffices finset_mem_Icc,
  exact { finset_Icc := λ a b, (h a b).to_finset,
          finset_mem_Icc := finset_mem_Icc },
  exact λ a b x, by rw [set.finite.mem_to_finset, set.mem_Icc],
end
Mario Carneiro (Sep 14 2021 at 19:31):
@Yaël Dillies
Yaël Dillies (Sep 14 2021 at 19:47):
Why can order_laws_tac work using the definition of ≤ whilefinset_Ico_laws_tac can't use finset_mem_Icc?
Yaël Dillies (Sep 14 2021 at 19:49):
Is what I'm trying to achieve that exotic?
Mario Carneiro (Sep 14 2021 at 19:52):
Because order_laws_tac doesn't need to reference anything outside its own statement for the proof, the proof is just rfl if you leave the default alone
Mario Carneiro (Sep 14 2021 at 19:53):
In your case, the proof for finset_mem_Ico depends on the proof of finset_mem_Icc
Mario Carneiro (Sep 14 2021 at 19:56):
I have a very hackish idea to get around this that would look for the current goal metavariable in the "result" (the term under construction), and hunt around in the parent of that expression to find the sibling proof of finset_mem_Ico
Yaël Dillies (Sep 14 2021 at 19:58):
That's the behavior I would have expected :smiley:
Yaël Dillies (Sep 14 2021 at 19:58):
because you can make fields dependent on others anyway, so that makes sense to be able to reference them.
Mario Carneiro (Sep 14 2021 at 20:00):
Here's a way to use spurious dependencies to make it work:
import data.set.finite
abbreviation id_annotate {α} (a : α) {β} (b : β) := b
theorem locally_finite_order.mem_Ico_of_mem_Icc
  {α : Type*} [preorder α] [decidable_rel ((≤) : α → α → Prop)]
  {finset_Icc : α → α → finset α}
  (finset_mem_Icc : ∀ a b x : α, x ∈ finset_Icc a b ↔ a ≤ x ∧ x ≤ b) :
  id_annotate finset_mem_Icc
    (∀ a b x : α, x ∈ (finset_Icc a b).filter (λ x, ¬b ≤ x) ↔ a ≤ x ∧ x < b) :=
λ a b x, by rw [finset.mem_filter, finset_mem_Icc, and_assoc, lt_iff_le_not_le]
meta def finset_Ico_laws_tac : tactic unit :=
`[exact locally_finite_order.mem_Ico_of_mem_Icc _]
class locally_finite_order (α : Type*) [preorder α] [decidable_rel ((≤) : α → α → Prop)] :=
(finset_Icc : α → α → finset α)
(finset_Ico : α → α → finset α := λ a b, (finset_Icc a b).filter (λ x, ¬b ≤ x))
(finset_mem_Icc : ∀ a b x : α, x ∈ finset_Icc a b ↔ a ≤ x ∧ x ≤ b)
(finset_mem_Ico : id_annotate finset_mem_Icc (∀ a b x : α, x ∈ finset_Ico a b ↔ a ≤ x ∧ x < b) . finset_Ico_laws_tac)
variables {α : Type*} [preorder α] [decidable_rel ((≤) : α → α → Prop)]
noncomputable def locally_finite_order_of_finite_Icc'
  (h : ∀ a b : α, (set.Icc a b).finite) :
  locally_finite_order α :=
{ finset_Icc := λ a b, (h a b).to_finset,
  finset_mem_Icc := λ a b x, by rw [set.finite.mem_to_finset, set.mem_Icc] }
Yaël Dillies (Sep 14 2021 at 20:04):
Ahah! The trick is to force finset_mem_Icc to appear in the context?
Yaël Dillies (Sep 14 2021 at 20:04):
You're a wizard, Mario. Thank you.
Mario Carneiro (Sep 14 2021 at 20:04):
in this case, we aren't putting it in the context, we're putting it in the type of the goal
Mario Carneiro (Sep 14 2021 at 20:05):
so lean can figure it out by unification
Yaël Dillies (Sep 14 2021 at 20:05):
I'm not sure I understand, but I'll keep that in mind for when I'll learn more about metaprogramming.
Mario Carneiro (Sep 14 2021 at 20:06):
If you actually want to prove finset_mem_Ico it is now uglified a bit, but autoparams also uglify the goal so I guess it's not that much worse
Mario Carneiro (Sep 14 2021 at 20:06):
this is actually pretty light on actual metaprogramming, this is more like elaborator-programming
Yaël Dillies (Sep 14 2021 at 20:06):
Can the abbreviation be made local?
Mario Carneiro (Sep 14 2021 at 20:07):
Actually I would probably want to lift it to init.core or logic.basic or so
Mario Carneiro (Sep 14 2021 at 20:07):
as you can see it's quite general
Mario Carneiro (Sep 14 2021 at 20:08):
But I didn't see an exact match among the annotation identity functions that lean has already
Yaël Dillies (Sep 14 2021 at 20:08):
Ah yeah, why not (even though it probably already exists?), but I was more thinking about stopping it from appearing in the goal.
Mario Carneiro (Sep 14 2021 at 20:08):
it's reducible so probably breathing lightly on it will make it go away
Mario Carneiro (Sep 14 2021 at 20:09):
in particular, if you want to prove that goal the first thing you do will probably be intros a b x and that will get rid of the junk
Yaël Dillies (Sep 14 2021 at 20:09):
What a metaphor. What else is there to scare it away?
Yaël Dillies (Sep 14 2021 at 20:09):
Ah yeah! then that's probably fine.
Yaël Dillies (Sep 14 2021 at 20:11):
Mario Carneiro said:
Actually I would probably want to lift it to
init.coreorlogic.basicor so
Do you want to do that? I have no idea how to name it nor where to put it further than what you said.
Mario Carneiro (Sep 14 2021 at 20:16):
Put it in the miscellaneous section of logic.basic for now, if you are working on a PR
Itai Bar-Natan (Sep 15 2021 at 13:35):
Perhaps it's possible to use something like ite to make the dependent field only take a default value if the base field is the default value? Something that looks roughly like
finset_mem_Ico : ite (finset_Ico = default_value)
  (opt_param (∀ a b x : α, x ∈ finset_Icc a b ↔ a ≤ x ∧ x ≤ b) (...))
  (∀ a b x : α, x ∈ finset_Icc a b ↔ a ≤ x ∧ x ≤ b)
I don't think ite is definitionally equal to the opt_param option and even if it is I'm worried the optional parameter mechanism won't evaluate the type to recognize opt_param, but maybe some modification of this (perhaps with the ". tactic" system that I haven't learned yet) can be used for a general mechanism for dependent optional parameters.
Yaël Dillies (Sep 15 2021 at 14:03):
This can't work like that because finset_Ico = default_value is always true for correct locally_finite_order declarations. = can't distinguish between propositional and definitional equality. But maybe you can instead put in a tactic that tries refl and changes branch depending on its success or failure?
Also note that an itecan't do it because you need the hypothesis finset_Ico = default_value to fill in the (...). You must use dite instead.
Last updated: May 02 2025 at 03:31 UTC