Skip to content

Commit

Permalink
comment out non-deterministic tests
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 4, 2024
1 parent 7729408 commit 1307193
Showing 1 changed file with 28 additions and 26 deletions.
54 changes: 28 additions & 26 deletions Test/Tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -150,29 +150,31 @@ theorem testBit_pred :
(Bool.xor ((List.range i).all fun j => ! testBit x j) (testBit x i))) := by
plausible

/--
error:
===================
Found a counter-example!
f := 1
issue: ULift.up 1 = ULift.up 0 does not hold
(1 shrinks)
-------------------
-/
#guard_msgs in
theorem ulift_nat (f : ULift.{1} Nat) : f = ⟨0⟩ := by
plausible

/--
error:
===================
Found a counter-example!
α := "ULift Int"
l := [0]
issue: [ULift.up 0] = [ULift.up 0, ULift.up 0] does not hold
(1 shrinks)
-------------------
-/
#guard_msgs in
theorem type_u (α : Type u) (l : List α) : l = l ++ l := by
plausible
-- FIXME: the following two tests have become non-deterministic.

-- /--
-- error:
-- ===================
-- Found a counter-example!
-- f := 1
-- issue: ULift.up 1 = ULift.up 0 does not hold
-- (1 shrinks)
-- -------------------
-- -/
-- #guard_msgs in
-- theorem ulift_nat (f : ULift.{1} Nat) : f = ⟨0⟩ := by
-- plausible

-- /--
-- error:
-- ===================
-- Found a counter-example!
-- α := "ULift Int"
-- l := [0]
-- issue: [ULift.up 0] = [ULift.up 0, ULift.up 0] does not hold
-- (1 shrinks)
-- -------------------
-- -/
-- #guard_msgs in
-- theorem type_u (α : Type u) (l : List α) : l = l ++ l := by
-- plausible

0 comments on commit 1307193

Please sign in to comment.