Skip to content

Commit 04a8e4a

Browse files
patch: Fix build
1 parent 1c4374e commit 04a8e4a

File tree

2 files changed

+3
-3
lines changed

2 files changed

+3
-3
lines changed

src/Iris/Algebra/CMRA.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1136,7 +1136,7 @@ theorem inc_iff {ma mb : Option α} :
11361136
· exact .inl Hmc.symm
11371137
· exact .inr ⟨_, Hmc⟩
11381138
· rintro (H|⟨_, _, _, _, (H|⟨z, _⟩)⟩) <;> subst_eqs
1139-
· exists mb; simp [op]
1139+
· exists mb
11401140
· exists none; simp [op]; exact H.symm
11411141
· exists some z
11421142

@@ -1147,7 +1147,7 @@ theorem incN_iff {ma mb : Option α} :
11471147
· exact .inl Hmc.symm
11481148
· exact .inr ⟨_, Hmc⟩
11491149
· rintro (H|⟨_, _, _, _, (H|⟨z, _⟩)⟩) <;> subst_eqs
1150-
· exists mb; simp [op]
1150+
· exists mb
11511151
· exists none; simp [op]; exact H.symm
11521152
· exists some z
11531153

src/Iris/Algebra/COFESolver.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -131,7 +131,7 @@ protected def Tower.embed (k) : A F k -n> Tower F := by
131131
rintro a _ eq rfl
132132
rw [Nat.add_assoc, Nat.add_left_cancel_iff] at eq; subst a
133133
apply down_up
134-
· cases (Nat.lt_or_eq_of_le h₁).resolve_left (h₂ ∘ Nat.lt_succ.1)
134+
· cases (Nat.lt_or_eq_of_le h₁).resolve_left (h₂ ∘ Nat.lt_succ_iff.1)
135135
have {a b} (e₁ : i+1+a = i+1) (e₂ : i+1 = i+b) :
136136
down F i (eqToHom e₁ (upN F a n)) ≡ downN F b (eqToHom e₂ n) := by
137137
cases Nat.add_left_cancel (k := 0) e₁; cases Nat.add_left_cancel e₂

0 commit comments

Comments
 (0)