Skip to content

Commit

Permalink
Update Set2.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
PratherConid committed Nov 5, 2023
1 parent e34568d commit b8f4ffd
Showing 1 changed file with 3 additions and 9 deletions.
12 changes: 3 additions & 9 deletions DuperOnMathlib/DuperOnMathlib/Set2.lean
Original file line number Diff line number Diff line change
Expand Up @@ -43,17 +43,15 @@ variable (s t u : Set α)
example (h : s ⊆ t) : s ∩ u ⊆ t ∩ u := by
auto [mem_inter_iff, subset_def, h]

set_option selFunction 3 in
-- zipperposition : Success
-- auto (raw duper) : Timeout
-- auto (portfolio duper) : Timeout
-- auto (portfolio duper) : Success
example : s ∩ (t ∪ u) ⊆ s ∩ t ∪ s ∩ u := by
auto [mem_inter_iff, mem_union, subset_def]

-- zipperposition : Success
-- auto (raw duper) : Timeout
-- auto (portfolio duper) : Timeout
set_option auto.native false in
-- auto (portfolio duper) : Success
example : s ∩ t ∪ s ∩ u ⊆ s ∩ (t ∪ u) := by
auto [mem_inter_iff, mem_union, subset_def]

Expand All @@ -68,7 +66,6 @@ example : (s \ t) \ u ⊆ s \ (t ∪ u) := by
-- zipperposition : Success
-- auto (raw duper) : Timeout
-- auto (portfolio duper) : Timeout
set_option auto.native false in
example : s ∩ t = t ∩ s := by
auto [Set.ext, mem_inter_iff]

Expand All @@ -81,7 +78,6 @@ example : s ∩ t = t ∩ s := by
-- zipperposition : Success
-- auto (raw duper) : Timeout
-- auto (portfolio duper) : Timeout
set_option auto.native false in
example : s ∩ (s ∪ t) = s := by
auto [Set.ext, mem_union, mem_inter_iff]

Expand All @@ -94,7 +90,6 @@ example : s ∩ (s ∪ t) = s := by
-- zipperposition : Success
-- auto (raw duper) : Timeout
-- auto (portfolio duper) : Timeout
set_option auto.native false in
example : s ∪ s ∩ t = s := by
auto [Set.ext, mem_union, mem_inter_iff]

Expand Down Expand Up @@ -124,8 +119,7 @@ example : s \ t ∪ t \ s = (s ∪ t) \ (s ∩ t) := by

-- zipperposition : Success
-- auto (raw duper) : Timeout
-- auto (portfolio duper) : Timeout
set_option auto.native false in
-- auto (portfolio duper) : Success
example : s \ t ∪ t \ s = (s ∪ t) \ (s ∩ t) := by
apply Set.ext; auto [mem_union, mem_inter_iff, mem_diff]

Expand Down

0 comments on commit b8f4ffd

Please sign in to comment.