Skip to content

Commit

Permalink
fix test
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Aug 25, 2024
1 parent d4d70e0 commit 9d72e4b
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion tests/lean/bool_simp.lean
Original file line number Diff line number Diff line change
Expand Up @@ -25,7 +25,7 @@ variable (u v w : Prop) [Decidable u] [Decidable v] [Decidable w]
#check_simp (true ≠ if u then b else c) ~> (if u then b = false else c = false)
#check_simp (u ∧ v → False) ~> u → v → False
#check_simp (u = (v ≠ w)) ~> (u ↔ ¬(v ↔ w))
#check_simp ((b = false) = (c = false)) ~> b = c
#check_simp ((b = false) = (c = false)) ~> (!b) = (!c)
#check_simp True ≠ (c = false) ~> c = true
#check_simp u ∧ u ∧ v ~> u ∧ v
#check_simp b || (b || c) ~> b || c
Expand Down

0 comments on commit 9d72e4b

Please sign in to comment.