Skip to content

Commit

Permalink
chore: post stage0 update fixups
Browse files Browse the repository at this point in the history
  • Loading branch information
collares committed Oct 23, 2023
1 parent 4e8cb97 commit 24fe58a
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion src/Init/Data/Nat/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -629,7 +629,7 @@ protected theorem sub_lt_sub_left : ∀ {k m n : Nat}, k < m → k < n → m - n
@[simp] protected theorem zero_sub (n : Nat) : 0 - n = 0 := by
induction n with
| zero => rfl
| succ n ih => simp [ih, Nat.sub_succ]
| succ n ih => simp only [ih, Nat.sub_succ]; decide

protected theorem sub_self_add (n m : Nat) : n - (n + m) = 0 := by
show (n + 0) - (n + m) = 0
Expand Down
2 changes: 1 addition & 1 deletion src/Init/SimpLemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -153,7 +153,7 @@ theorem Bool.or_assoc (a b c : Bool) : (a || b || c) = (a || (b || c)) := by
@[simp] theorem bne_self_eq_false' [DecidableEq α] (a : α) : (a != a) = false := by simp [bne]

@[simp] theorem Nat.le_zero_eq (a : Nat) : (a ≤ 0) = (a = 0) :=
propext ⟨fun h => Nat.le_antisymm h (Nat.zero_le ..), fun h => by simp [h]⟩
propext ⟨fun h => Nat.le_antisymm h (Nat.zero_le ..), fun h => by rw [h]; decide

@[simp] theorem decide_False : decide False = false := rfl
@[simp] theorem decide_True : decide True = true := rfl
Expand Down
2 changes: 1 addition & 1 deletion src/Lean/Compiler/LCNF/PassManager.lean
Original file line number Diff line number Diff line change
Expand Up @@ -46,7 +46,7 @@ structure Pass where
Resulting phase.
-/
phaseOut : Phase := phase
phaseInv : phaseOut ≥ phase := by simp
phaseInv : phaseOut ≥ phase := by simp_arith
/--
The name of the `Pass`
-/
Expand Down

0 comments on commit 24fe58a

Please sign in to comment.