Skip to content

Commit

Permalink
Replace original namespace with open in pseudoelts
Browse files Browse the repository at this point in the history
  • Loading branch information
adomani committed May 30, 2023
1 parent ffaa865 commit 48471f3
Showing 1 changed file with 1 addition and 3 deletions.
4 changes: 1 addition & 3 deletions counterexamples/pseudoelement.lean
Expand Up @@ -35,7 +35,7 @@ namespace counterexample

noncomputable theory

namespace category_theory.abelian.pseudoelement
open category_theory.abelian.pseudoelement

/-- `x` is given by `t ↦ (t, 2 * t)`. -/
def x : over ((of ℤ ℚ) ⊞ (of ℤ ℚ)) :=
Expand Down Expand Up @@ -121,6 +121,4 @@ lemma exist_ne_and_fst_eq_fst_and_snd_eq_snd : ∃ x y : (of ℤ ℚ) ⊞ (of
(biprod.snd : (of ℤ ℚ) ⊞ (of ℤ ℚ) ⟶ _) x = (biprod.snd : (of ℤ ℚ) ⊞ (of ℤ ℚ) ⟶ _) y:=
⟨⟦x⟧, ⟦y⟧, mk_x_ne_mk_y, fst_mk_x_eq_fst_mk_y, snd_mk_x_eq_snd_mk_y⟩

end category_theory.abelian.pseudoelement

end counterexample

0 comments on commit 48471f3

Please sign in to comment.