Skip to content

Commit 8cc4435

Browse files
committed
chore: more adaptations for lean4#5542
In [lean4#5542](leanprover/lean4#5542) we are deprecating `inductive ... :=`, `structure ... :=`, and `class ... :=` for their `... where` counterparts. Continuation of #17655.
1 parent 1fb2cbc commit 8cc4435

File tree

2 files changed

+2
-2
lines changed

2 files changed

+2
-2
lines changed

Diff for: test/Simps.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -101,7 +101,7 @@ infix:25 (priority := default+1) " ≃ " => Equiv'
101101

102102
/- Since `prod` and `PProd` are a special case for `@[simps]`, we define a new structure to test
103103
the basic functionality.-/
104-
structure MyProd (α β : Type _) := (fst : α) (snd : β)
104+
structure MyProd (α β : Type _) where (fst : α) (snd : β)
105105

106106
def MyProd.map {α α' β β'} (f : α → α') (g : β → β') (x : MyProd α β) : MyProd α' β' :=
107107
⟨f x.1, g x.2

Diff for: test/Traversable.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -34,7 +34,7 @@ inductive RecData (α : Type u) : Type u
3434

3535
#guard_msgs (drop info) in #synth LawfulTraversable RecData
3636

37-
unsafe structure MetaStruct (α : Type u) : Type u :=
37+
unsafe structure MetaStruct (α : Type u) : Type u where
3838
x : α
3939
y : ℤ
4040
z : List α

0 commit comments

Comments
 (0)