Skip to content

Commit

Permalink
Add another example to temp2.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
JOSHCLUNE committed Oct 12, 2024
1 parent e435720 commit 92c1afd
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions Duper/Tests/temp2.lean
Original file line number Diff line number Diff line change
Expand Up @@ -107,3 +107,11 @@ theorem forall₂_true_iff1 {β : α → Sort} : (∀ a, β a → True) ↔ True

-- Look into why Duper can solve `forall₂_true_iff1` but not `forall₂_true_iff2`
theorem forall₂_true_iff2 {β : α → Sort _} : (∀ a, β a → True) ↔ True := by duper [*]

--------------------------------------------------------------------
set_option trace.duper.saturate.debug true in
set_option duper.throwPortfolioErrors true in
theorem exists₂_comm
{ι₁ ι₂ : Sort} {κ₁ : ι₁ → Sort} {κ₂ : ι₂ → Sort} {p : ∀ i₁, κ₁ i₁ → ∀ i₂, κ₂ i₂ → Prop} :
(∃ i₁ j₁ i₂ j₂, p i₁ j₁ i₂ j₂) ↔ ∃ i₂ j₂ i₁ j₁, p i₁ j₁ i₂ j₂ := by
duper [*] {preprocessing := no_preprocessing}

0 comments on commit 92c1afd

Please sign in to comment.