Skip to content

Commit

Permalink
test: for rw with nonDependentFirst
Browse files Browse the repository at this point in the history
  • Loading branch information
leodemoura authored and kim-em committed Jun 23, 2024
1 parent 464813e commit 034cad9
Showing 1 changed file with 14 additions and 0 deletions.
14 changes: 14 additions & 0 deletions tests/lean/run/rw_nondepFirst.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,14 @@
def Set (ι : Type) := ι → Prop

namespace Set

def univ : Set ι := fun _ => True
def empty : Set ι := fun _ => False

def pi {ι : Type} {α : ι → Type} (s : Set ι) (t : (i : ι) → Set (α i)) : Set ((i : ι) → α i) := sorry

theorem univ_pi_eq_empty (ht : t i = empty) : Set.pi univ t = empty := sorry

example (i : ι) (h : t i = empty) : Set.pi univ t = empty := by
rw [univ_pi_eq_empty]
· exact h

0 comments on commit 034cad9

Please sign in to comment.