diff --git a/src/logic/basic.lean b/src/logic/basic.lean index 571a140f04b96..0dbc7530909b1 100644 --- a/src/logic/basic.lean +++ b/src/logic/basic.lean @@ -215,6 +215,16 @@ lemma fact_iff {p : Prop} : fact p ↔ p := ⟨λ h, h.1, λ h, ⟨h⟩⟩ Π i₂ j₂ i₁ j₁, φ i₁ j₁ i₂ j₂ := λ i₂ j₂ i₁ j₁, f i₁ j₁ i₂ j₂ +/-- If `x : α . tac_name` then `x.out : α`. These are definitionally equal, but this can +nevertheless be useful for various reasons, e.g. to apply further projection notation or in an +argument to `simp`. -/ +def auto_param.out {α : Sort*} {n : name} (x : auto_param α n) : α := x + +/-- If `x : α := d` then `x.out : α`. These are definitionally equal, but this can +nevertheless be useful for various reasons, e.g. to apply further projection notation or in an +argument to `simp`. -/ +def opt_param.out {α : Sort*} {d : α} (x : α := d) : α := x + end miscellany open function