Skip to content

Commit

Permalink
Adding another skolem issue to bugs.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
JOSHCLUNE committed Nov 1, 2023
1 parent 6fb53b8 commit 8c7553b
Showing 1 changed file with 15 additions and 0 deletions.
15 changes: 15 additions & 0 deletions Duper/Tests/bugs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -88,3 +88,18 @@ argument has type
but function has type
Type u_2 → Type u_2
-/

-- Bug 8
set_option trace.Saturate.debug true in
example (h1 : ∀ x : Nat, x > 0 → ∃ y : Fin x, y.1 = 0) (h2 : 3 > 0) : ∃ z : Fin 3, z.1 = 0 := by
duper [h1, h2]

/-
The final active set contains both of the following clauses:
- ∀ (a : Fin 3), a.1 ≠ 0
- ∀ (a : Fin 3), (skS.0 Type 0 ((x_0 : Nat) → Fin x_0 → Fin x_0) 3 a).1 = 0
If it were possible to unify `a` from the first clause with `(skS.0 Type 0 ((x_0 : Nat) → Fin x_0 → Fin x_0) 3 a)` from
the second clause, then duper would be able to derive a contradiction. However, the current manner in which skolem symbols
are constructed prevents this.
-/

0 comments on commit 8c7553b

Please sign in to comment.