File tree Expand file tree Collapse file tree 2 files changed +6
-1
lines changed Expand file tree Collapse file tree 2 files changed +6
-1
lines changed Original file line number Diff line number Diff line change @@ -78,7 +78,7 @@ end Elab.Tactic.Ext
78
78
end Lean
79
79
80
80
attribute [ext] Prod PProd Sigma PSigma
81
- attribute [ext] funext propext Subtype.eq
81
+ attribute [ext] funext propext Subtype.eq Array.ext
82
82
83
83
@[ext] protected theorem PUnit.ext (x y : PUnit) : x = y := rfl
84
84
protected theorem Unit.ext (x y : Unit) : x = y := rfl
Original file line number Diff line number Diff line change @@ -82,6 +82,11 @@ example (f : ℕ × (ℕ → ℕ)) : f = f := by
82
82
example (f : Empty → Empty) : f = f := by
83
83
ext ⟨⟩
84
84
85
+ example (xs : Array α) : xs.map id = xs := by
86
+ ext
87
+ . simp
88
+ . simp
89
+
85
90
@[ext (iff := false)] theorem ext_intros {n m : Nat} (w : ∀ n m : Nat, n = m) : n = m := by apply w
86
91
87
92
#guard_msgs (drop warning) in
You can’t perform that action at this time.
0 commit comments